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

add lemmas 'intuitionistic' and 'intuitionistically_intro'

parent 3cb65333
No related branches found
No related tags found
No related merge requests found
...@@ -1431,9 +1431,19 @@ Proof. by rewrite -(persistent_persistently P) persistently_and_sep_assoc. Qed. ...@@ -1431,9 +1431,19 @@ Proof. by rewrite -(persistent_persistently P) persistently_and_sep_assoc. Qed.
Lemma impl_wand_2 P `{!Persistent P} Q : (P -∗ Q) P Q. Lemma impl_wand_2 P `{!Persistent P} Q : (P -∗ Q) P Q.
Proof. apply impl_intro_l. by rewrite persistent_and_sep_1 wand_elim_r. Qed. Proof. apply impl_intro_l. by rewrite persistent_and_sep_1 wand_elim_r. Qed.
(** We don't have a [Intuitionistic] typeclass, but if we did, this
would be its only field. *)
Lemma intuitionistic P `{!Persistent P, !Affine P} : P P.
Proof. rewrite intuitionistic_intuitionistically. done. Qed.
Section persistent_bi_absorbing. Section persistent_bi_absorbing.
Context `{BiAffine PROP}. Context `{BiAffine PROP}.
Lemma intuitionistically_intro P Q `{!Persistent P} : (P Q) P Q.
Proof.
intros HP. rewrite (persistent P) HP intuitionistically_into_persistently //.
Qed.
Lemma persistent_and_sep P Q `{HPQ : !TCOr (Persistent P) (Persistent Q)} : Lemma persistent_and_sep P Q `{HPQ : !TCOr (Persistent P) (Persistent Q)} :
P Q ⊣⊢ P Q. P Q ⊣⊢ P Q.
Proof. Proof.
......
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