Documentation

Mathlib.Init.Propext

Additional congruence lemmas.

theorem imp_congr_eq {a : Prop} {b : Prop} {c : Prop} {d : Prop} (h₁ : a = c) (h₂ : b = d) :
(ab) = (cd)
theorem imp_congr_ctx_eq {a : Prop} {b : Prop} {c : Prop} {d : Prop} (h₁ : a = c) (h₂ : cb = d) :
(ab) = (cd)
theorem eq_true_intro {a : Prop} (h : a) :
theorem eq_false_intro {a : Prop} (h : ¬a) :
theorem Iff.to_eq {a : Prop} {b : Prop} (h : a b) :
a = b
theorem iff_eq_eq {a : Prop} {b : Prop} :
(a b) = (a = b)