Documentation

Mathlib.Order.Nat

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 #

@[simp]
theorem Nat.bot_eq_zero :
= 0
theorem Nat.isLeast_find {p : Prop} [DecidablePred p] (hp : ∃ (n : ), p n) :
IsLeast {n : | p n} (Nat.find hp)

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.