mathlib documentation

algebra.group_with_zero.power

Powers of elements of groups with an adjoined zero element #

In this file we define integer power functions for groups with an adjoined zero element. This generalises the integer power function on a division ring.

@[simp]
theorem zero_pow' {M : Type u_1} [monoid_with_zero M] (n : ) :
n 00 ^ n = 0
theorem ne_zero_pow {M : Type u_1} [monoid_with_zero M] {a : M} {n : } (hn : n 0) :
a ^ n 0a 0
@[simp]
theorem zero_pow_eq_zero {M : Type u_1} [monoid_with_zero M] [nontrivial M] {n : } :
0 ^ n = 0 0 < n
theorem ring.inverse_pow {M : Type u_1} [monoid_with_zero M] (r : M) (n : ) :
@[simp]
theorem inv_pow₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a⁻¹ ^ n = (a ^ n)⁻¹
theorem pow_sub₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) {m n : } (ha : a 0) (h : n m) :
a ^ (m - n) = (a ^ m) * (a ^ n)⁻¹
theorem pow_sub_of_lt {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) {m n : } (h : n < m) :
a ^ (m - n) = (a ^ m) * (a ^ n)⁻¹
theorem pow_inv_comm₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (m n : ) :
(a⁻¹ ^ m) * a ^ n = (a ^ n) * a⁻¹ ^ m
theorem inv_pow_sub₀ {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} {m n : } (ha : a 0) (h : n m) :
a⁻¹ ^ (m - n) = (a ^ m)⁻¹ * a ^ n
theorem inv_pow_sub_of_lt {G₀ : Type u_1} [group_with_zero G₀] {m n : } (a : G₀) (h : n < m) :
a⁻¹ ^ (m - n) = (a ^ m)⁻¹ * a ^ n
@[simp]
theorem one_zpow₀ {G₀ : Type u_1} [group_with_zero G₀] (n : ) :
1 ^ n = 1
theorem zero_zpow {G₀ : Type u_1} [group_with_zero G₀] (z : ) :
z 00 ^ z = 0
theorem zero_zpow_eq {G₀ : Type u_1} [group_with_zero G₀] (n : ) :
0 ^ n = ite (n = 0) 1 0
@[simp]
theorem zpow_neg₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a ^ -n = (a ^ n)⁻¹
theorem mul_zpow_neg_one₀ {G₀ : Type u_1} [group_with_zero G₀] (a b : G₀) :
(a * b) ^ -1 = (b ^ -1) * a ^ -1
theorem zpow_neg_one₀ {G₀ : Type u_1} [group_with_zero G₀] (x : G₀) :
x ^ -1 = x⁻¹
theorem inv_zpow₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a⁻¹ ^ n = (a ^ n)⁻¹
theorem zpow_add_one₀ {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (ha : a 0) (n : ) :
a ^ (n + 1) = (a ^ n) * a
theorem zpow_sub_one₀ {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (ha : a 0) (n : ) :
a ^ (n - 1) = (a ^ n) * a⁻¹
theorem zpow_add₀ {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (ha : a 0) (m n : ) :
a ^ (m + n) = (a ^ m) * a ^ n
theorem zpow_add' {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} {m n : } (h : a 0 m + n 0 m = 0 n = 0) :
a ^ (m + n) = (a ^ m) * a ^ n
theorem zpow_one_add₀ {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (h : a 0) (i : ) :
a ^ (1 + i) = a * a ^ i
theorem semiconj_by.zpow_right₀ {G₀ : Type u_1} [group_with_zero G₀] {a x y : G₀} (h : semiconj_by a x y) (m : ) :
semiconj_by a (x ^ m) (y ^ m)
theorem commute.zpow_right₀ {G₀ : Type u_1} [group_with_zero G₀] {a b : G₀} (h : commute a b) (m : ) :
commute a (b ^ m)
theorem commute.zpow_left₀ {G₀ : Type u_1} [group_with_zero G₀] {a b : G₀} (h : commute a b) (m : ) :
commute (a ^ m) b
theorem commute.zpow_zpow₀ {G₀ : Type u_1} [group_with_zero G₀] {a b : G₀} (h : commute a b) (m n : ) :
commute (a ^ m) (b ^ n)
theorem commute.zpow_self₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
commute (a ^ n) a
theorem commute.self_zpow₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
commute a (a ^ n)
theorem commute.zpow_zpow_self₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (m n : ) :
commute (a ^ m) (a ^ n)
theorem zpow_bit0₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a ^ bit0 n = (a ^ n) * a ^ n
theorem zpow_bit1₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a ^ bit1 n = ((a ^ n) * a ^ n) * a
theorem zpow_mul₀ {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (m n : ) :
a ^ m * n = (a ^ m) ^ n
theorem zpow_mul₀' {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (m n : ) :
a ^ m * n = (a ^ n) ^ m
@[simp, norm_cast]
theorem units.coe_zpow₀ {G₀ : Type u_1} [group_with_zero G₀] (u : G₀ˣ) (n : ) :
(u ^ n) = u ^ n
theorem zpow_ne_zero_of_ne_zero {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (ha : a 0) (z : ) :
a ^ z 0
theorem zpow_sub₀ {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (ha : a 0) (z1 z2 : ) :
a ^ (z1 - z2) = a ^ z1 / a ^ z2
theorem commute.mul_zpow₀ {G₀ : Type u_1} [group_with_zero G₀] {a b : G₀} (h : commute a b) (i : ) :
(a * b) ^ i = (a ^ i) * b ^ i
theorem zpow_bit0' {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a ^ bit0 n = (a * a) ^ n
theorem zpow_bit1' {G₀ : Type u_1} [group_with_zero G₀] (a : G₀) (n : ) :
a ^ bit1 n = ((a * a) ^ n) * a
theorem zpow_eq_zero {G₀ : Type u_1} [group_with_zero G₀] {x : G₀} {n : } (h : x ^ n = 0) :
x = 0
theorem zpow_eq_zero_iff {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} {n : } (hn : 0 < n) :
a ^ n = 0 a = 0
theorem zpow_ne_zero {G₀ : Type u_1} [group_with_zero G₀] {x : G₀} (n : ) :
x 0x ^ n 0
theorem zpow_neg_mul_zpow_self {G₀ : Type u_1} [group_with_zero G₀] (n : ) {x : G₀} (h : x 0) :
(x ^ -n) * x ^ n = 1
theorem one_div_pow {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (n : ) :
(1 / a) ^ n = 1 / a ^ n
theorem one_div_zpow {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (n : ) :
(1 / a) ^ n = 1 / a ^ n
@[simp]
theorem inv_zpow' {G₀ : Type u_1} [group_with_zero G₀] {a : G₀} (n : ) :
a⁻¹ ^ n = a ^ -n
@[simp]
theorem div_pow {G₀ : Type u_1} [comm_group_with_zero G₀] (a b : G₀) (n : ) :
(a / b) ^ n = a ^ n / b ^ n
theorem mul_zpow₀ {G₀ : Type u_1} [comm_group_with_zero G₀] (a b : G₀) (m : ) :
(a * b) ^ m = (a ^ m) * b ^ m
@[simp]
theorem div_zpow₀ {G₀ : Type u_1} [comm_group_with_zero G₀] (a : G₀) {b : G₀} (n : ) :
(a / b) ^ n = a ^ n / b ^ n
theorem div_sq_cancel {G₀ : Type u_1} [comm_group_with_zero G₀] (a b : G₀) :
(a ^ 2) * b / a = a * b
def zpow_group_hom₀ {G₀ : Type u_1} [comm_group_with_zero G₀] (n : ) :
G₀ →* G₀

The n-th power map (n an integer) on a commutative group with zero, considered as a group homomorphism.

Equations
theorem monoid_with_zero_hom.map_zpow {G₀ : Type u_1} {G₀' : Type u_2} [group_with_zero G₀] [group_with_zero G₀'] (f : G₀ →*₀ G₀') (x : G₀) (n : ) :
f (x ^ n) = f x ^ n

If a monoid homomorphism f between two group_with_zeros maps 0 to 0, then it maps x^n, n : ℤ, to (f x)^n.

theorem pow_minus_two_nonneg {R : Type u_1} [linear_ordered_field R] {a : R} :
0 a ^ -2