diff --git a/theories/bi/embedding.v b/theories/bi/embedding.v index 3ddb3479a35f461e932dbdc51e2c9e561416d8a4..3eaa91784100ffdc0e859c0b2e8fffe90df61878 100644 --- a/theories/bi/embedding.v +++ b/theories/bi/embedding.v @@ -84,7 +84,7 @@ Section embed_laws. Proof. eapply bi_embed_mixin_ne, bi_embed_mixin. Qed. Global Instance embed_mono : Proper ((⊢) ==> (⊢)) embed. Proof. eapply bi_embed_mixin_mono, bi_embed_mixin. Qed. - Lemma embed_emp_valid_inj P : ( ⊢@{PROP2} ⎡P⎤) → ⊢ P. + Lemma embed_emp_valid_inj P : (⊢@{PROP2} ⎡P⎤) → ⊢ P. Proof. eapply bi_embed_mixin_emp_valid_inj, bi_embed_mixin. Qed. Lemma embed_emp_2 : emp ⊢ ⎡emp⎤. Proof. eapply bi_embed_mixin_emp_2, bi_embed_mixin. Qed. diff --git a/theories/bi/interface.v b/theories/bi/interface.v index f233be208ce53d5d2be95fb674ef2aef1d1b1773..9fb540cffcab6b35feda93b38e7f0a708957a937 100644 --- a/theories/bi/interface.v +++ b/theories/bi/interface.v @@ -262,7 +262,7 @@ Instance bi_inhabited {PROP : bi} : Inhabited PROP := populate (bi_pure True). Notation "P ⊢ Q" := (bi_entails P%I Q%I) : stdpp_scope. Notation "P ⊢@{ PROP } Q" := (bi_entails (PROP:=PROP) P%I Q%I) (only parsing) : stdpp_scope. Notation "(⊢)" := bi_entails (only parsing) : stdpp_scope. -Notation "(⊢@{ PROP } )" := (bi_entails (PROP:=PROP)) (only parsing) : stdpp_scope. +Notation "('⊢@{' PROP } )" := (bi_entails (PROP:=PROP)) (only parsing) : stdpp_scope. Notation "P ⊣⊢ Q" := (equiv (A:=bi_car _) P%I Q%I) : stdpp_scope. Notation "P ⊣⊢@{ PROP } Q" := (equiv (A:=bi_car PROP) P%I Q%I) (only parsing) : stdpp_scope.