Documentation

Mathlib.Algebra.Order.Group.Nat

The naturals form a linear ordered monoid #

This file contains the linear ordered monoid instance on the natural numbers.

See note [foundational algebra order theory].

Instances #

Equations
  • One or more equations did not get rendered due to their size.
Equations
Equations
  • One or more equations did not get rendered due to their size.

Miscellaneous lemmas #

theorem NeZero.one_le {n : } [NeZero n] :
1 n
theorem Nat.pow_left_strictMono {n : } (hn : n 0) :
StrictMono fun (x : ) => x ^ n

See also pow_left_strictMonoOn.

theorem StrictMono.nat_pow {α : Type u_1} {n : } {f : α} [Preorder α] (hn : n 0) (hf : StrictMono f) :
StrictMono fun (x : α) => f x ^ n