Documentation

Init.Omega.Logic

Specializations of basic logic lemmas #

These are useful for omega while constructing proofs, but not considered generally useful so are hidden in the Lean.Omega namespace.

If you find yourself needing them elsewhere, please move them first to another file.

theorem Lean.Omega.and_not_not_of_not_or {p : Prop} {q : Prop} (h : ¬(p q)) :
theorem Lean.Omega.Decidable.and_not_of_not_imp {a : Prop} {b : Prop} [Decidable a] (h : ¬(ab)) :
a ¬b
theorem Lean.Omega.ite_disjunction {α : Type u} {P : Prop} [Decidable P] {a : α} {b : α} :
P (if P then a else b) = a ¬P (if P then a else b) = b