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

prove later commuting around equality one way

parent a2f75cd0
No related branches found
No related tags found
No related merge requests found
......@@ -167,6 +167,12 @@ Qed.
Lemma later_equivI {A : ofeT} (x y : A) : Next x Next y ⊣⊢ (x y).
Proof. apply (anti_symm _); auto using later_eq_1, later_eq_2. Qed.
Lemma later_equivI_prop (P Q : PROP) : (P Q) ( P) ( Q).
Proof.
move: (@later_contractive PROP)=> /contractive_alt [g [? Hlt]].
rewrite (Hlt P) (Hlt Q) -later_equivI.
eapply (internal_eq_rewrite' (Next P) (Next Q) (λ Qx, g (Next P) g Qx)%I); auto.
Qed.
(* Later derived *)
Hint Resolve later_mono : core.
......
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