mathlib3 documentation

algebra.group_power.order

Lemmas about the interaction of power operations with order #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Note that some lemmas are in algebra/group_power/lemmas.lean as they import files which depend on this file.

theorem pow_le_pow_of_le_left' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] [covariant_class M M (function.swap has_mul.mul) has_le.le] {a b : M} (hab : a b) (i : ) :
a ^ i b ^ i
theorem one_le_pow_of_one_le' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {a : M} (H : 1 a) (n : ) :
1 a ^ n
theorem nsmul_nonneg {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {a : M} (H : 0 a) (n : ) :
0 n a
theorem pow_le_one' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {a : M} (H : a 1) (n : ) :
a ^ n 1
theorem nsmul_nonpos {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {a : M} (H : a 0) (n : ) :
n a 0
theorem pow_le_pow' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {a : M} {n m : } (ha : 1 a) (h : n m) :
a ^ n a ^ m
theorem nsmul_le_nsmul {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {a : M} {n m : } (ha : 0 a) (h : n m) :
n a m a
theorem nsmul_le_nsmul_of_nonpos {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {a : M} {n m : } (ha : a 0) (h : n m) :
m a n a
theorem pow_le_pow_of_le_one' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {a : M} {n m : } (ha : a 1) (h : n m) :
a ^ m a ^ n
theorem one_lt_pow' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {a : M} (ha : 1 < a) {k : } (hk : k 0) :
1 < a ^ k
theorem nsmul_pos {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {a : M} (ha : 0 < a) {k : } (hk : k 0) :
0 < k a
theorem pow_lt_one' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {a : M} (ha : a < 1) {k : } (hk : k 0) :
a ^ k < 1
theorem nsmul_neg {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {a : M} (ha : a < 0) {k : } (hk : k 0) :
k a < 0
theorem pow_lt_pow' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] [covariant_class M M has_mul.mul has_lt.lt] {a : M} {n m : } (ha : 1 < a) (h : n < m) :
a ^ n < a ^ m
theorem nsmul_lt_nsmul {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] [covariant_class M M has_add.add has_lt.lt] {a : M} {n m : } (ha : 0 < a) (h : n < m) :
n a < m a
theorem nsmul_strict_mono_right {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] [covariant_class M M has_add.add has_lt.lt] {a : M} (ha : 0 < a) :
strict_mono (λ (ᾰ : ), a)
theorem left.one_le_pow_of_le {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {x : M} (hx : 1 x) {n : } :
1 x ^ n
theorem left.pow_nonneg {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {x : M} (hx : 0 x) {n : } :
0 n x
theorem left.pow_le_one_of_le {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_le.le] {x : M} (hx : x 1) {n : } :
x ^ n 1
theorem left.pow_nonpos {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_le.le] {x : M} (hx : x 0) {n : } :
n x 0
theorem right.one_le_pow_of_le {M : Type u_4} [monoid M] [preorder M] [covariant_class M M (function.swap has_mul.mul) has_le.le] {x : M} (hx : 1 x) {n : } :
1 x ^ n
theorem right.pow_nonneg {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M (function.swap has_add.add) has_le.le] {x : M} (hx : 0 x) {n : } :
0 n x
theorem right.pow_nonpos {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M (function.swap has_add.add) has_le.le] {x : M} (hx : x 0) {n : } :
n x 0
theorem right.pow_le_one_of_le {M : Type u_4} [monoid M] [preorder M] [covariant_class M M (function.swap has_mul.mul) has_le.le] {x : M} (hx : x 1) {n : } :
x ^ n 1
theorem strict_mono.pow_right' {β : Type u_1} {M : Type u_4} [monoid M] [preorder M] [preorder β] [covariant_class M M has_mul.mul has_lt.lt] [covariant_class M M (function.swap has_mul.mul) has_lt.lt] {f : β M} (hf : strict_mono f) {n : } :
n 0 strict_mono (λ (a : β), f a ^ n)
theorem strict_mono.nsmul_left {β : Type u_1} {M : Type u_4} [add_monoid M] [preorder M] [preorder β] [covariant_class M M has_add.add has_lt.lt] [covariant_class M M (function.swap has_add.add) has_lt.lt] {f : β M} (hf : strict_mono f) {n : } :
n 0 strict_mono (λ (a : β), n f a)
@[nolint]
theorem pow_strict_mono_right' {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_lt.lt] [covariant_class M M (function.swap has_mul.mul) has_lt.lt] {n : } (hn : n 0) :
strict_mono (λ (a : M), a ^ n)

See also pow_strict_mono_right

@[nolint]
theorem monotone.pow_right {β : Type u_1} {M : Type u_4} [monoid M] [preorder M] [preorder β] [covariant_class M M has_mul.mul has_le.le] [covariant_class M M (function.swap has_mul.mul) has_le.le] {f : β M} (hf : monotone f) (n : ) :
monotone (λ (a : β), f a ^ n)
theorem monotone.nsmul_left {β : Type u_1} {M : Type u_4} [add_monoid M] [preorder M] [preorder β] [covariant_class M M has_add.add has_le.le] [covariant_class M M (function.swap has_add.add) has_le.le] {f : β M} (hf : monotone f) (n : ) :
monotone (λ (a : β), n f a)
theorem left.pow_neg {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M has_add.add has_lt.lt] {n : } {x : M} (hn : 0 < n) (h : x < 0) :
n x < 0
theorem left.pow_lt_one_of_lt {M : Type u_4} [monoid M] [preorder M] [covariant_class M M has_mul.mul has_lt.lt] {n : } {x : M} (hn : 0 < n) (h : x < 1) :
x ^ n < 1
theorem right.pow_lt_one_of_lt {M : Type u_4} [monoid M] [preorder M] [covariant_class M M (function.swap has_mul.mul) has_lt.lt] {n : } {x : M} (hn : 0 < n) (h : x < 1) :
x ^ n < 1
theorem right.pow_neg {M : Type u_4} [add_monoid M] [preorder M] [covariant_class M M (function.swap has_add.add) has_lt.lt] {n : } {x : M} (hn : 0 < n) (h : x < 0) :
n x < 0
theorem nsmul_nonneg_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] {x : M} {n : } (hn : n 0) :
0 n x 0 x
theorem one_le_pow_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] {x : M} {n : } (hn : n 0) :
1 x ^ n 1 x
theorem nsmul_nonpos_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] {x : M} {n : } (hn : n 0) :
n x 0 x 0
theorem pow_le_one_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] {x : M} {n : } (hn : n 0) :
x ^ n 1 x 1
theorem one_lt_pow_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] {x : M} {n : } (hn : n 0) :
1 < x ^ n 1 < x
theorem nsmul_pos_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] {x : M} {n : } (hn : n 0) :
0 < n x 0 < x
theorem pow_lt_one_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] {x : M} {n : } (hn : n 0) :
x ^ n < 1 x < 1
theorem nsmul_neg_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] {x : M} {n : } (hn : n 0) :
n x < 0 x < 0
theorem pow_eq_one_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] {x : M} {n : } (hn : n 0) :
x ^ n = 1 x = 1
theorem nsmul_eq_zero_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] {x : M} {n : } (hn : n 0) :
n x = 0 x = 0
theorem nsmul_le_nsmul_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] [covariant_class M M has_add.add has_lt.lt] {a : M} {m n : } (ha : 0 < a) :
m a n a m n
theorem pow_le_pow_iff' {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] [covariant_class M M has_mul.mul has_lt.lt] {a : M} {m n : } (ha : 1 < a) :
a ^ m a ^ n m n
theorem nsmul_lt_nsmul_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_le.le] [covariant_class M M has_add.add has_lt.lt] {a : M} {m n : } (ha : 0 < a) :
m a < n a m < n
theorem pow_lt_pow_iff' {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] [covariant_class M M has_mul.mul has_lt.lt] {a : M} {m n : } (ha : 1 < a) :
a ^ m < a ^ n m < n
theorem le_of_pow_le_pow' {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_lt.lt] [covariant_class M M (function.swap has_mul.mul) has_lt.lt] {a b : M} {n : } (hn : n 0) :
a ^ n b ^ n a b
theorem left.nsmul_neg_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M has_add.add has_lt.lt] {n : } {x : M} (hn : 0 < n) :
n x < 0 x < 0
theorem left.pow_lt_one_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_lt.lt] {n : } {x : M} (hn : 0 < n) :
x ^ n < 1 x < 1
theorem right.pow_lt_one_iff {M : Type u_4} [monoid M] [linear_order M] [covariant_class M M (function.swap has_mul.mul) has_lt.lt] {n : } {x : M} (hn : 0 < n) :
x ^ n < 1 x < 1
theorem right.nsmul_neg_iff {M : Type u_4} [add_monoid M] [linear_order M] [covariant_class M M (function.swap has_add.add) has_lt.lt] {n : } {x : M} (hn : 0 < n) :
n x < 0 x < 0
theorem one_le_zpow {G : Type u_3} [div_inv_monoid G] [preorder G] [covariant_class G G has_mul.mul has_le.le] {x : G} (H : 1 x) {n : } (hn : 0 n) :
1 x ^ n
theorem zsmul_nonneg {G : Type u_3} [sub_neg_monoid G] [preorder G] [covariant_class G G has_add.add has_le.le] {x : G} (H : 0 x) {n : } (hn : 0 n) :
0 n x
theorem canonically_ordered_comm_semiring.pow_pos {R : Type u_5} [canonically_ordered_comm_semiring R] {a : R} (H : 0 < a) (n : ) :
0 < a ^ n
theorem zero_pow_le_one {R : Type u_5} [ordered_semiring R] (n : ) :
0 ^ n 1
theorem pow_add_pow_le {R : Type u_5} [ordered_semiring R] {x y : R} {n : } (hx : 0 x) (hy : 0 y) (hn : n 0) :
x ^ n + y ^ n (x + y) ^ n
theorem pow_le_one {R : Type u_5} [ordered_semiring R] {a : R} (n : ) (h₀ : 0 a) (h₁ : a 1) :
a ^ n 1
theorem pow_lt_one {R : Type u_5} [ordered_semiring R] {a : R} (h₀ : 0 a) (h₁ : a < 1) {n : } (hn : n 0) :
a ^ n < 1
theorem one_le_pow_of_one_le {R : Type u_5} [ordered_semiring R] {a : R} (H : 1 a) (n : ) :
1 a ^ n
theorem pow_mono {R : Type u_5} [ordered_semiring R] {a : R} (h : 1 a) :
monotone (λ (n : ), a ^ n)
theorem pow_le_pow {R : Type u_5} [ordered_semiring R] {a : R} {n m : } (ha : 1 a) (h : n m) :
a ^ n a ^ m
theorem le_self_pow {R : Type u_5} [ordered_semiring R] {a : R} {m : } (ha : 1 a) (h : m 0) :
a a ^ m
theorem pow_le_pow_of_le_left {R : Type u_5} [ordered_semiring R] {a b : R} (ha : 0 a) (hab : a b) (i : ) :
a ^ i b ^ i
theorem one_lt_pow {R : Type u_5} [ordered_semiring R] {a : R} (ha : 1 < a) {n : } (hn : n 0) :
1 < a ^ n
theorem pow_lt_pow_of_lt_left {R : Type u_5} [strict_ordered_semiring R] {x y : R} (h : x < y) (hx : 0 x) {n : } :
0 < n x ^ n < y ^ n
theorem strict_mono_on_pow {R : Type u_5} [strict_ordered_semiring R] {n : } (hn : 0 < n) :
strict_mono_on (λ (x : R), x ^ n) (set.Ici 0)
theorem pow_strict_mono_right {R : Type u_5} [strict_ordered_semiring R] {a : R} (h : 1 < a) :
strict_mono (λ (n : ), a ^ n)
theorem pow_lt_pow {R : Type u_5} [strict_ordered_semiring R] {a : R} {n m : } (h : 1 < a) (h2 : n < m) :
a ^ n < a ^ m
theorem pow_lt_pow_iff {R : Type u_5} [strict_ordered_semiring R] {a : R} {n m : } (h : 1 < a) :
a ^ n < a ^ m n < m
theorem pow_le_pow_iff {R : Type u_5} [strict_ordered_semiring R] {a : R} {n m : } (h : 1 < a) :
a ^ n a ^ m n m
theorem strict_anti_pow {R : Type u_5} [strict_ordered_semiring R] {a : R} (h₀ : 0 < a) (h₁ : a < 1) :
strict_anti (λ (n : ), a ^ n)
theorem pow_lt_pow_iff_of_lt_one {R : Type u_5} [strict_ordered_semiring R] {a : R} {n m : } (h₀ : 0 < a) (h₁ : a < 1) :
a ^ m < a ^ n n < m
theorem pow_lt_pow_of_lt_one {R : Type u_5} [strict_ordered_semiring R] {a : R} (h : 0 < a) (ha : a < 1) {i j : } (hij : i < j) :
a ^ j < a ^ i
theorem pow_lt_self_of_lt_one {R : Type u_5} [strict_ordered_semiring R] {a : R} {n : } (h₀ : 0 < a) (h₁ : a < 1) (hn : 1 < n) :
a ^ n < a
theorem sq_pos_of_pos {R : Type u_5} [strict_ordered_semiring R] {a : R} (ha : 0 < a) :
0 < a ^ 2
theorem pow_bit0_pos_of_neg {R : Type u_5} [strict_ordered_ring R] {a : R} (ha : a < 0) (n : ) :
0 < a ^ bit0 n
theorem pow_bit1_neg {R : Type u_5} [strict_ordered_ring R] {a : R} (ha : a < 0) (n : ) :
a ^ bit1 n < 0
theorem sq_pos_of_neg {R : Type u_5} [strict_ordered_ring R] {a : R} (ha : a < 0) :
0 < a ^ 2
theorem pow_le_one_iff_of_nonneg {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) {n : } (hn : n 0) :
a ^ n 1 a 1
theorem one_le_pow_iff_of_nonneg {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) {n : } (hn : n 0) :
1 a ^ n 1 a
theorem one_lt_pow_iff_of_nonneg {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) {n : } (hn : n 0) :
1 < a ^ n 1 < a
theorem pow_lt_one_iff_of_nonneg {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) {n : } (hn : n 0) :
a ^ n < 1 a < 1
theorem sq_le_one_iff {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) :
a ^ 2 1 a 1
theorem sq_lt_one_iff {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) :
a ^ 2 < 1 a < 1
theorem one_le_sq_iff {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) :
1 a ^ 2 1 a
theorem one_lt_sq_iff {R : Type u_5} [linear_ordered_semiring R] {a : R} (ha : 0 a) :
1 < a ^ 2 1 < a
@[simp]
theorem pow_left_inj {R : Type u_5} [linear_ordered_semiring R] {x y : R} {n : } (Hxpos : 0 x) (Hypos : 0 y) (Hnpos : 0 < n) :
x ^ n = y ^ n x = y
theorem lt_of_pow_lt_pow {R : Type u_5} [linear_ordered_semiring R] {a b : R} (n : ) (hb : 0 b) (h : a ^ n < b ^ n) :
a < b
theorem le_of_pow_le_pow {R : Type u_5} [linear_ordered_semiring R] {a b : R} (n : ) (hb : 0 b) (hn : 0 < n) (h : a ^ n b ^ n) :
a b
@[simp]
theorem sq_eq_sq {R : Type u_5} [linear_ordered_semiring R] {a b : R} (ha : 0 a) (hb : 0 b) :
a ^ 2 = b ^ 2 a = b
theorem lt_of_mul_self_lt_mul_self {R : Type u_5} [linear_ordered_semiring R] {a b : R} (hb : 0 b) :
a * a < b * b a < b
theorem pow_abs {R : Type u_5} [linear_ordered_ring R] (a : R) (n : ) :
|a| ^ n = |a ^ n|
theorem abs_neg_one_pow {R : Type u_5} [linear_ordered_ring R] (n : ) :
|(-1) ^ n| = 1
theorem abs_pow_eq_one {R : Type u_5} [linear_ordered_ring R] (a : R) {n : } (h : 0 < n) :
|a ^ n| = 1 |a| = 1
theorem pow_bit0_nonneg {R : Type u_5} [linear_ordered_ring R] (a : R) (n : ) :
0 a ^ bit0 n
theorem sq_nonneg {R : Type u_5} [linear_ordered_ring R] (a : R) :
0 a ^ 2
theorem pow_two_nonneg {R : Type u_5} [linear_ordered_ring R] (a : R) :
0 a ^ 2

Alias of sq_nonneg.

theorem pow_bit0_pos {R : Type u_5} [linear_ordered_ring R] {a : R} (h : a 0) (n : ) :
0 < a ^ bit0 n
theorem sq_pos_of_ne_zero {R : Type u_5} [linear_ordered_ring R] (a : R) (h : a 0) :
0 < a ^ 2
theorem pow_two_pos_of_ne_zero {R : Type u_5} [linear_ordered_ring R] (a : R) (h : a 0) :
0 < a ^ 2

Alias of sq_pos_of_ne_zero.

theorem pow_bit0_pos_iff {R : Type u_5} [linear_ordered_ring R] (a : R) {n : } (hn : n 0) :
0 < a ^ bit0 n a 0
theorem sq_pos_iff {R : Type u_5} [linear_ordered_ring R] (a : R) :
0 < a ^ 2 a 0
theorem sq_abs {R : Type u_5} [linear_ordered_ring R] (x : R) :
|x| ^ 2 = x ^ 2
theorem abs_sq {R : Type u_5} [linear_ordered_ring R] (x : R) :
|x ^ 2| = x ^ 2
theorem sq_lt_sq {R : Type u_5} [linear_ordered_ring R] {x y : R} :
x ^ 2 < y ^ 2 |x| < |y|
theorem sq_lt_sq' {R : Type u_5} [linear_ordered_ring R] {x y : R} (h1 : -y < x) (h2 : x < y) :
x ^ 2 < y ^ 2
theorem sq_le_sq {R : Type u_5} [linear_ordered_ring R] {x y : R} :
x ^ 2 y ^ 2 |x| |y|
theorem sq_le_sq' {R : Type u_5} [linear_ordered_ring R] {x y : R} (h1 : -y x) (h2 : x y) :
x ^ 2 y ^ 2
theorem abs_lt_of_sq_lt_sq {R : Type u_5} [linear_ordered_ring R] {x y : R} (h : x ^ 2 < y ^ 2) (hy : 0 y) :
|x| < y
theorem abs_lt_of_sq_lt_sq' {R : Type u_5} [linear_ordered_ring R] {x y : R} (h : x ^ 2 < y ^ 2) (hy : 0 y) :
-y < x x < y
theorem abs_le_of_sq_le_sq {R : Type u_5} [linear_ordered_ring R] {x y : R} (h : x ^ 2 y ^ 2) (hy : 0 y) :
|x| y
theorem abs_le_of_sq_le_sq' {R : Type u_5} [linear_ordered_ring R] {x y : R} (h : x ^ 2 y ^ 2) (hy : 0 y) :
-y x x y
theorem sq_eq_sq_iff_abs_eq_abs {R : Type u_5} [linear_ordered_ring R] (x y : R) :
x ^ 2 = y ^ 2 |x| = |y|
@[simp]
theorem sq_le_one_iff_abs_le_one {R : Type u_5} [linear_ordered_ring R] (x : R) :
x ^ 2 1 |x| 1
@[simp]
theorem sq_lt_one_iff_abs_lt_one {R : Type u_5} [linear_ordered_ring R] (x : R) :
x ^ 2 < 1 |x| < 1
@[simp]
theorem one_le_sq_iff_one_le_abs {R : Type u_5} [linear_ordered_ring R] (x : R) :
1 x ^ 2 1 |x|
@[simp]
theorem one_lt_sq_iff_one_lt_abs {R : Type u_5} [linear_ordered_ring R] (x : R) :
1 < x ^ 2 1 < |x|
theorem pow_four_le_pow_two_of_pow_two_le {R : Type u_5} [linear_ordered_ring R] {x y : R} (h : x ^ 2 y) :
x ^ 4 y ^ 2
theorem two_mul_le_add_sq {R : Type u_5} [linear_ordered_comm_ring R] (a b : R) :
2 * a * b a ^ 2 + b ^ 2

Arithmetic mean-geometric mean (AM-GM) inequality for linearly ordered commutative rings.

theorem two_mul_le_add_pow_two {R : Type u_5} [linear_ordered_comm_ring R] (a b : R) :
2 * a * b a ^ 2 + b ^ 2

Alias of two_mul_le_add_sq.

theorem pow_pos_iff {M : Type u_4} [linear_ordered_comm_monoid_with_zero M] [no_zero_divisors M] {a : M} {n : } (hn : 0 < n) :
0 < a ^ n 0 < a
theorem pow_lt_pow_succ {M : Type u_4} [linear_ordered_comm_group_with_zero M] {a : M} {n : } (ha : 1 < a) :
a ^ n < a ^ n.succ
theorem pow_lt_pow₀ {M : Type u_4} [linear_ordered_comm_group_with_zero M] {a : M} {m n : } (ha : 1 < a) (hmn : m < n) :
a ^ m < a ^ n
theorem monoid_hom.map_neg_one {M : Type u_4} {R : Type u_5} [ring R] [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] (f : R →* M) :
f (-1) = 1
@[simp]
theorem monoid_hom.map_neg {M : Type u_4} {R : Type u_5} [ring R] [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] (f : R →* M) (x : R) :
f (-x) = f x
theorem monoid_hom.map_sub_swap {M : Type u_4} {R : Type u_5} [ring R] [monoid M] [linear_order M] [covariant_class M M has_mul.mul has_le.le] (f : R →* M) (x y : R) :
f (x - y) = f (y - x)