Skip to content
Snippets Groups Projects
Verified Commit e5a2bcff authored by Paolo G. Giarrusso's avatar Paolo G. Giarrusso
Browse files

sbi_internal_eq: add "sections" of notation, following stdpp

parent ab3b5c77
No related branches found
No related tags found
No related merge requests found
...@@ -5,6 +5,10 @@ Section tests. ...@@ -5,6 +5,10 @@ Section tests.
Context {PROP : sbi}. Context {PROP : sbi}.
Implicit Types P Q R : PROP. Implicit Types P Q R : PROP.
Lemma type_sbi_internal_eq_annot P :
P ≡@{PROP} P (≡@{PROP}) P P (P .) P (. P) P.
Proof. done. Qed.
Lemma test_eauto_emp_isplit_biwand P : emp P ∗-∗ P. Lemma test_eauto_emp_isplit_biwand P : emp P ∗-∗ P.
Proof. eauto 6. Qed. Proof. eauto 6. Qed.
......
...@@ -290,6 +290,12 @@ Notation "∃ x .. y , P" := ...@@ -290,6 +290,12 @@ Notation "∃ x .. y , P" :=
Notation "'<pers>' P" := (bi_persistently P) : bi_scope. Notation "'<pers>' P" := (bi_persistently P) : bi_scope.
Infix "≡" := sbi_internal_eq : bi_scope. Infix "≡" := sbi_internal_eq : bi_scope.
Infix "≡@{ A }" := (sbi_internal_eq (A := A)) (only parsing) : bi_scope.
Notation "( X ≡.)" := (sbi_internal_eq X) (only parsing) : bi_scope.
Notation "(.≡ X )" := (λ Y, Y X)%I (only parsing) : bi_scope.
Notation "(≡@{ A } )" := (sbi_internal_eq (A := A)) (only parsing) : bi_scope.
Notation "▷ P" := (sbi_later P) : bi_scope. Notation "▷ P" := (sbi_later P) : bi_scope.
Definition bi_emp_valid {PROP : bi} (P : PROP) : Prop := emp P. Definition bi_emp_valid {PROP : bi} (P : PROP) : Prop := emp P.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment