Skip to content

Commit

Permalink
progress on 32-bit examples
Browse files Browse the repository at this point in the history
  • Loading branch information
mansky1 committed Mar 22, 2024
1 parent 30d2510 commit ed06891
Show file tree
Hide file tree
Showing 58 changed files with 8,928 additions and 1,573 deletions.
4 changes: 4 additions & 0 deletions floyd/Funspec_old_Notation.v
Original file line number Diff line number Diff line change
@@ -0,0 +1,4 @@
Require Export VST.floyd.funspec_old.

Global Close Scope funspec_scope.
Global Open Scope old_funspec_scope.
5 changes: 4 additions & 1 deletion floyd/compat.v
Original file line number Diff line number Diff line change
@@ -1,10 +1,11 @@
Require Import VST.veric.SequentialClight.
Require Import VST.floyd.proofauto.

Export Unset SsrRewrite.
#[export] Unset SsrRewrite.

Notation assert := (@assert (VSTΣ unit)).
Notation funspec := (@funspec (VSTΣ unit)).
Notation funspecs := (@funspecs (VSTΣ unit)).

(* Concrete instance of the Iris typeclasses for no ghost state or external calls *)
#[local] Instance default_pre : VSTGpreS unit (VSTΣ unit) := subG_VSTGpreS _.
Expand Down Expand Up @@ -54,6 +55,8 @@ Ltac simplify_func_tycontext' DD ::=

Notation "P |-- Q" := (P ⊢ Q)
(at level 99, Q at level 200, right associativity, only parsing) : stdpp_scope.
Notation " 'ENTAIL' d ',' P |-- Q " :=
(@bi_entails (monPredI environ_index (iPropI _)) (local (tc_environ d) ∧ P%assert) Q%assert) (at level 99, P at level 98, Q at level 98).
Notation "'!!' φ" := (bi_pure φ%type%stdpp) (at level 15) : bi_scope.
Notation "P && Q" := (P ∧ Q)%I (only parsing) : bi_scope.
Notation "P || Q" := (P ∨ Q)%I (only parsing) : bi_scope.
Expand Down
Loading

0 comments on commit ed06891

Please sign in to comment.