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

show that persistently and affinely-persistently are fixpoints of something

parent 985f9713
No related branches found
No related tags found
No related merge requests found
...@@ -842,6 +842,14 @@ Proof. ...@@ -842,6 +842,14 @@ Proof.
- by rewrite (affinely_elim_emp P) left_id affinely_elim. - by rewrite (affinely_elim_emp P) left_id affinely_elim.
Qed. Qed.
Lemma persistently_alt_fixpoint P :
<pers> P ⊣⊢ P <pers> P.
Proof.
apply (anti_symm _).
- rewrite -persistently_and_sep_elim. apply and_intro; done.
- rewrite comm persistently_absorbing. done.
Qed.
Lemma persistently_wand P Q : <pers> (P -∗ Q) <pers> P -∗ <pers> Q. Lemma persistently_wand P Q : <pers> (P -∗ Q) <pers> P -∗ <pers> Q.
Proof. apply wand_intro_r. by rewrite persistently_sep_2 wand_elim_l. Qed. Proof. apply wand_intro_r. by rewrite persistently_sep_2 wand_elim_l. Qed.
...@@ -962,6 +970,17 @@ Proof. ...@@ -962,6 +970,17 @@ Proof.
- apply impl_intro_l. by rewrite persistently_and_affinely_sep_l wand_elim_r. - apply impl_intro_l. by rewrite persistently_and_affinely_sep_l wand_elim_r.
Qed. Qed.
Lemma affinely_persistently_alt_fixpoint P :
P ⊣⊢ emp (P P).
Proof.
apply (anti_symm ()).
- apply and_intro; first exact: affinely_elim_emp.
rewrite {1}affinely_persistently_sep_dup. apply sep_mono; last done.
apply affinely_persistently_elim.
- apply and_mono; first done. rewrite {2}persistently_alt_fixpoint.
apply sep_mono; first done. apply and_elim_r.
Qed.
(* Conditional affinely modality *) (* Conditional affinely modality *)
Global Instance affinely_if_ne p : NonExpansive (@bi_affinely_if PROP p). Global Instance affinely_if_ne p : NonExpansive (@bi_affinely_if PROP p).
Proof. solve_proper. Qed. Proof. solve_proper. 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