-- I actually thought that ∀p, ∃q, (q ≠ p) ∧ q! -- However, propositional extensionality tells us that (p ↔ q) → p = q theorem finiteTrueProps : ¬∀p, ∃q, (q ≠ p) ∧ q := by intro h have := h True simp at this theorem finiteFalseProps : ¬∀p, ∃q, (q ≠ p) ∧ ¬q := by intro h have := h False simp at this