Power operations on monoids and groups #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The power operation on monoids and groups.
We separate this from group, because it depends on ℕ
,
which in turn depends on other parts of algebra.
This module contains lemmas about a ^ n
and n • a
, where n : ℕ
or n : ℤ
.
Further lemmas can be found in algebra.group_power.lemmas
.
The analogous results for groups with zero can be found in algebra.group_with_zero.power
.
Notation #
a ^ n
is used as notation forhas_pow.pow a n
; in this filen : ℕ
orn : ℤ
.n • a
is used as notation forhas_smul.smul n a
; in this filen : ℕ
orn : ℤ
.
Implementation details #
We adopt the convention that 0^0 = 1
.
Commutativity #
First we prove some facts about semiconj_by
and commute
. They do not require any theory about
pow
and/or nsmul
and will be useful later in this file.
Commutative (additive) monoid #
Multiplication by a natural n
on a commutative additive
monoid, considered as a morphism of additive monoids.
The n
th power map on a commutative monoid for a natural n
, considered as a morphism of
monoids.
The n
-th power map (for an integer n
) on a commutative group, considered as a group
homomorphism.
Multiplication by an integer n
on a commutative additive group, considered as an
additive group homomorphism.