bookshelf/Common/Nat/Basic.lean

13 lines
237 B
Plaintext
Raw Permalink Normal View History

2023-08-08 14:56:13 +00:00
import Mathlib.Data.Set.Basic
import Mathlib.Tactic.NormNum
2023-08-08 14:56:13 +00:00
namespace Nat
/--
If `n < m⁺`, then `n < m` or `n = m`.
-/
theorem lt_or_eq_of_lt {n m : Nat} (h : n < m.succ) : n < m n = m :=
lt_or_eq_of_le (lt_succ.mp h)
2023-12-14 19:49:31 +00:00
end Nat