From 49530cb3a19856d287d638bbc74530f380503c42 Mon Sep 17 00:00:00 2001 From: Ralf Jung <jung@mpi-sws.org> Date: Tue, 10 Mar 2020 18:12:26 +0100 Subject: [PATCH] rename later_equivI_prop for consistency --- theories/bi/derived_laws_sbi.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) diff --git a/theories/bi/derived_laws_sbi.v b/theories/bi/derived_laws_sbi.v index 098d145b4..a20d4191e 100644 --- a/theories/bi/derived_laws_sbi.v +++ b/theories/bi/derived_laws_sbi.v @@ -172,7 +172,7 @@ 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). +Lemma later_equivI_prop_2 (P Q : PROP) : ▷ (P ≡ Q) ⊢ (▷ P) ≡ (▷ Q). Proof. apply (f_equiv_contractive _). Qed. (* Later derived *) -- GitLab