simple-counterexamples/SimpleCounterexamples/BadInfinities.lean
2025-04-08 22:31:48 -04:00

18 lines
511 B
Text
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

abbrev HasInfinity (α : Type) [LT α] := ∃(inf : α), ∀n, n < inf
theorem lt_irrefl_imp_no_infinity
(α : Type) [LT α] (irrefl : ∀(n : α), ¬n < n) : ¬HasInfinity α := by
intro h
have ⟨inf, h⟩ := h
have hlt : inf < inf := h inf
exact irrefl inf hlt
theorem no_nat_infinity : ¬HasInfinity Nat :=
lt_irrefl_imp_no_infinity Nat Nat.lt_irrefl
theorem no_int_infinity : ¬HasInfinity Nat :=
lt_irrefl_imp_no_infinity Nat Nat.lt_irrefl
-- it's… not difficult to see the pattern