diff --git a/algebra/upred.v b/algebra/upred.v index 73d521139463509343e82842df645fa8ad66e1e9..6072149717cad4add9421669ba4a36eafe5d7a47 100644 --- a/algebra/upred.v +++ b/algebra/upred.v @@ -564,6 +564,8 @@ Proof. intros ->; apply iff_refl. Qed. Lemma pure_mono φ1 φ2 : (φ1 → φ2) → ■φ1 ⊢ ■φ2. Proof. intros; apply pure_elim with φ1; eauto using pure_intro. Qed. +Lemma pure_iff φ1 φ2 : (φ1 ↔ φ2) → ■φ1 ⊣⊢ ■φ2. +Proof. intros [??]; apply (anti_symm _); auto using pure_mono. Qed. Lemma and_mono P P' Q Q' : (P ⊢ Q) → (P' ⊢ Q') → P ∧ P' ⊢ Q ∧ Q'. Proof. auto. Qed. Lemma and_mono_l P P' Q : (P ⊢ Q) → P ∧ P' ⊢ Q ∧ P'.