Skip to content
Snippets Groups Projects
Commit 101c4e5d authored by Ralf Jung's avatar Ralf Jung
Browse files

lemmas about □?p P and <affine>?p P

parent 7af1bbd3
No related branches found
No related tags found
No related merge requests found
...@@ -1181,6 +1181,9 @@ Proof. destruct p; simpl; auto using intuitionistically_sep. Qed. ...@@ -1181,6 +1181,9 @@ Proof. destruct p; simpl; auto using intuitionistically_sep. Qed.
Lemma intuitionistically_if_idemp p P : ?p ?p P ⊣⊢ ?p P. Lemma intuitionistically_if_idemp p P : ?p ?p P ⊣⊢ ?p P.
Proof. destruct p; simpl; auto using intuitionistically_idemp. Qed. Proof. destruct p; simpl; auto using intuitionistically_idemp. Qed.
Lemma intuitionistically_if_unfold p P : ?p P ⊣⊢ <affine>?p <pers>?p P.
Proof. by destruct p. Qed.
(* Properties of persistent propositions *) (* Properties of persistent propositions *)
Global Instance Persistent_proper : Proper (() ==> iff) (@Persistent PROP). Global Instance Persistent_proper : Proper (() ==> iff) (@Persistent PROP).
Proof. solve_proper. Qed. Proof. solve_proper. Qed.
...@@ -1288,6 +1291,8 @@ Global Instance sep_affine P Q : Affine P → Affine Q → Affine (P ∗ Q). ...@@ -1288,6 +1291,8 @@ Global Instance sep_affine P Q : Affine P → Affine Q → Affine (P ∗ Q).
Proof. rewrite /Affine=>-> ->. by rewrite left_id. Qed. Proof. rewrite /Affine=>-> ->. by rewrite left_id. Qed.
Global Instance affinely_affine P : Affine (<affine> P). Global Instance affinely_affine P : Affine (<affine> P).
Proof. rewrite /bi_affinely. apply _. Qed. Proof. rewrite /bi_affinely. apply _. Qed.
Global Instance affinely_if_affine p P : Affine P Affine (<affine>?p P).
Proof. destruct p; simpl; apply _. Qed.
Global Instance intuitionistically_affine P : Affine ( P). Global Instance intuitionistically_affine P : Affine ( P).
Proof. rewrite /bi_intuitionistically. apply _. Qed. Proof. rewrite /bi_intuitionistically. apply _. Qed.
......
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