Skip to content
Snippets Groups Projects
Commit b433bf12 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Add lemma `intuitionistically_impl_wand_2 P Q : □ (P -∗ Q) ⊢ □ (P → Q)`.

This lemma is similar to `persistently_impl_wand_2`.
parent af5e50e7
No related branches found
No related tags found
No related merge requests found
......@@ -1094,6 +1094,9 @@ Proof.
apply sep_mono; first done. apply and_elim_r.
Qed.
Lemma intuitionistically_impl_wand_2 P Q : (P -∗ Q) (P Q).
Proof. by rewrite /bi_intuitionistically persistently_impl_wand_2. Qed.
Lemma impl_alt P Q : (P Q) ⊣⊢ R, R <pers> (P R -∗ Q).
Proof.
apply (anti_symm ()).
......
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