The natural numbers form a linear order #
This file contains the linear order instance on the natural numbers.
See note [foundational algebra order theory].
TODO #
Move the LinearOrder ℕ
instance here (https://github.com/leanprover-community/mathlib4/pull/13092).
Miscellaneous lemmas #
Nat.find
is the minimum natural number satisfying a predicate p
.
theorem
Set.Nonempty.isLeast_natFind
{s : Set ℕ}
[DecidablePred fun (x : ℕ) => x ∈ s]
(hs : s.Nonempty)
:
Nat.find
is the minimum element of a nonempty set of natural numbers.