diff --git a/theories/bi/derived_laws_sbi.v b/theories/bi/derived_laws_sbi.v index 098d145b492586d2fdff26bdbffe5cb5f70be7e4..a20d4191ea58f56b47c2c33645cb9215327dbac9 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 *)