Lemmas about power operations on monoids and groups
This file contains lemmas about monoid.pow
, group.pow
, nsmul
, gsmul
which require additional imports besides those available in .basic
.
(Additive) monoid
Bernoulli's inequality for n : ℕ
, -2 ≤ a
.
Bernoulli's inequality reformulated to estimate a^n
.
Monoid homomorphisms from multiplicative ℕ
are defined by the image
of multiplicative.of_add 1
.
Equations
- powers_hom M = {to_fun := λ (x : M), {to_fun := λ (n : multiplicative ℕ), x ^ n.to_add, map_one' := _, map_mul' := _}, inv_fun := λ (f : multiplicative ℕ →* M), ⇑f (multiplicative.of_add 1), left_inv := _, right_inv := _}
Monoid homomorphisms from multiplicative ℤ
are defined by the image
of multiplicative.of_add 1
.
Equations
- gpowers_hom G = {to_fun := λ (x : G), {to_fun := λ (n : multiplicative ℤ), x ^ n.to_add, map_one' := _, map_mul' := _}, inv_fun := λ (f : multiplicative ℤ →* G), ⇑f (multiplicative.of_add 1), left_inv := _, right_inv := _}
Additive homomorphisms from ℕ
are defined by the image of 1
.
Additive homomorphisms from ℤ
are defined by the image of 1
.
Commutativity (again)
Facts about semiconj_by
and commute
that require gpow
or gsmul
, or the fact that integer
multiplication equals semiring multiplication.
Moving to the opposite monoid commutes with taking powers.