Basic lemmas about ordered rings #
theorem
IsSquare.nonneg
{R : Type u_3}
[Semiring R]
[LinearOrder R]
[IsRightCancelAdd R]
[ZeroLEOneClass R]
[ExistsAddOfLE R]
[PosMulMono R]
[AddLeftStrictMono R]
{x : R}
(h : IsSquare x)
:
theorem
MonoidHom.map_neg_one
{M : Type u_2}
{R : Type u_3}
[Ring R]
[Monoid M]
[LinearOrder M]
[MulLeftMono M]
(f : R →* M)
:
@[simp]
theorem
MonoidHom.map_neg
{M : Type u_2}
{R : Type u_3}
[Ring R]
[Monoid M]
[LinearOrder M]
[MulLeftMono M]
(f : R →* M)
(x : R)
:
@[deprecated mul_le_one₀ (since := "2024-09-28")]
theorem
mul_le_one
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a b : M₀}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
(ha : a ≤ 1)
(hb₀ : 0 ≤ b)
(hb : b ≤ 1)
:
Alias of mul_le_one₀
.
@[deprecated pow_le_one₀ (since := "2024-09-28")]
theorem
pow_le_one
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a : M₀}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
{n : ℕ}
:
Alias of pow_le_one₀
.
@[deprecated pow_lt_one₀ (since := "2024-09-28")]
theorem
pow_lt_one
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a : M₀}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
(h₀ : 0 ≤ a)
(h₁ : a < 1)
{n : ℕ}
:
Alias of pow_lt_one₀
.
@[deprecated one_le_pow₀ (since := "2024-09-28")]
theorem
one_le_pow_of_one_le
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a : M₀}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
(ha : 1 ≤ a)
{n : ℕ}
:
Alias of one_le_pow₀
.
@[deprecated one_lt_pow₀ (since := "2024-09-28")]
theorem
one_lt_pow
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a : M₀}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
(ha : 1 < a)
{n : ℕ}
:
Alias of one_lt_pow₀
.
@[deprecated pow_right_mono₀ (since := "2024-10-04")]
theorem
pow_right_mono
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a : M₀}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
(h : 1 ≤ a)
:
Alias of pow_right_mono₀
.
@[deprecated pow_le_pow_right₀ (since := "2024-10-04")]
theorem
pow_le_pow_right
{M₀ : Type u_1}
[MonoidWithZero M₀]
[Preorder M₀]
{a : M₀}
{m n : ℕ}
[ZeroLEOneClass M₀]
[PosMulMono M₀]
[MulPosMono M₀]
(ha : 1 ≤ a)
(hmn : m ≤ n)
:
Alias of pow_le_pow_right₀
.
@[reducible, inline]
abbrev
OrderedRing.toStrictOrderedRing
(α : Type u_4)
[OrderedRing α]
[NoZeroDivisors α]
[Nontrivial α]
:
Turn an ordered domain into a strict ordered ring.
Instances For
@[deprecated pow_right_strictMono₀ (since := "2024-11-13")]
theorem
pow_right_strictMono
{R : Type u_3}
[StrictOrderedSemiring R]
{a : R}
(h : 1 < a)
:
StrictMono fun (x : ℕ) => a ^ x
@[deprecated pow_right_strictAnti₀ (since := "2024-11-13")]
theorem
pow_right_strictAnti
{R : Type u_3}
[StrictOrderedSemiring R]
{a : R}
(h₀ : 0 < a)
(h₁ : a < 1)
:
StrictAnti fun (x : ℕ) => a ^ x
@[deprecated pow_right_injective₀ (since := "2024-11-12")]
theorem
pow_right_injective
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
(ha₀ : 0 < a)
(ha₁ : a ≠ 1)
:
Function.Injective fun (x : ℕ) => a ^ x
Lemmas for canonically linear ordered semirings or linear ordered rings #
The slightly unusual typeclass assumptions [LinearOrderedSemiring R] [ExistsAddOfLE R]
cover two
more familiar settings:
[LinearOrderedRing R]
, egℤ
,ℚ
orℝ
[CanonicallyLinearOrderedSemiring R]
(although we don't actually have this typeclass), egℕ
,ℚ≥0
orℝ≥0
theorem
Even.pow_nonneg
{R : Type u_3}
[LinearOrderedSemiring R]
{n : ℕ}
[ExistsAddOfLE R]
(hn : Even n)
(a : R)
:
theorem
Even.pow_pos
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Even n)
(ha : a ≠ 0)
:
theorem
Odd.pow_neg_iff
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
theorem
Odd.pow_nonneg_iff
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
theorem
Odd.pow_nonpos_iff
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
theorem
Odd.pow_pos_iff
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
theorem
Odd.pow_nonpos
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
Alias of the reverse direction of Odd.pow_nonpos_iff
.
theorem
Odd.pow_neg
{R : Type u_3}
[LinearOrderedSemiring R]
{a : R}
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
Alias of the reverse direction of Odd.pow_neg_iff
.
theorem
Odd.strictMono_pow
{R : Type u_3}
[LinearOrderedSemiring R]
{n : ℕ}
[ExistsAddOfLE R]
(hn : Odd n)
:
StrictMono fun (a : R) => a ^ n
Alias of the reverse direction of sq_pos_iff
.
Alias of the reverse direction of sq_pos_iff
.
Alias of the reverse direction of sq_pos_iff
.
theorem
pow_four_le_pow_two_of_pow_two_le
{R : Type u_3}
[LinearOrderedSemiring R]
{a b : R}
[ExistsAddOfLE R]
(h : a ^ 2 ≤ b)
: