Powers of elements of groups with an adjoined zero element #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
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.
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 : ℤ) :
theorem
commute.zpow_left₀
{G₀ : Type u_1}
[group_with_zero G₀]
{a b : G₀}
(h : commute a b)
(m : ℤ) :
theorem
commute.zpow_zpow₀
{G₀ : Type u_1}
[group_with_zero G₀]
{a b : G₀}
(h : commute a b)
(m n : ℤ) :
theorem
zpow_ne_zero_of_ne_zero
{G₀ : Type u_1}
[group_with_zero G₀]
{a : G₀}
(ha : a ≠ 0)
(z : ℤ) :
@[simp]
theorem
map_zpow₀
{F : Type u_1}
{G₀ : Type u_2}
{G₀' : Type u_3}
[group_with_zero G₀]
[group_with_zero G₀']
[monoid_with_zero_hom_class F G₀ G₀']
(f : F)
(x : G₀)
(n : ℤ) :
If a monoid homomorphism f
between two group_with_zero
s maps 0
to 0
, then it maps x^n
,
n : ℤ
, to (f x)^n
.