Skip to content
Snippets Groups Projects
Commit 2dc55133 authored by Jacques-Henri Jourdan's avatar Jacques-Henri Jourdan
Browse files

pure_flip_mono

parent 873f2d0a
No related branches found
No related tags found
No related merge requests found
...@@ -236,6 +236,8 @@ Lemma pure_mono φ1 φ2 : (φ1 → φ2) → ⌜φ1⌝ ⊢ ⌜φ2⌝. ...@@ -236,6 +236,8 @@ Lemma pure_mono φ1 φ2 : (φ1 → φ2) → ⌜φ1⌝ ⊢ ⌜φ2⌝.
Proof. intros; apply pure_elim with φ1; eauto. Qed. Proof. intros; apply pure_elim with φ1; eauto. Qed.
Global Instance pure_mono' : Proper (impl ==> ()) (@uPred_pure M). Global Instance pure_mono' : Proper (impl ==> ()) (@uPred_pure M).
Proof. intros φ1 φ2; apply pure_mono. Qed. Proof. intros φ1 φ2; apply pure_mono. Qed.
Global Instance pure_flip_mono : Proper (flip impl ==> flip ()) (@uPred_pure M).
Proof. intros φ1 φ2; apply pure_mono. Qed.
Lemma pure_iff φ1 φ2 : (φ1 φ2) φ1 ⊣⊢ φ2⌝. Lemma pure_iff φ1 φ2 : (φ1 φ2) φ1 ⊣⊢ φ2⌝.
Proof. intros [??]; apply (anti_symm _); auto using pure_mono. Qed. Proof. intros [??]; apply (anti_symm _); auto using pure_mono. Qed.
Lemma pure_intro_l φ Q R : φ (φ Q R) Q R. Lemma pure_intro_l φ Q R : φ (φ Q R) Q R.
......
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