Endomorphisms, homomorphisms and group actions #
This file defines Function.End
as the monoid of endomorphisms on a type,
and provides results relating group actions with these endomorphisms.
Notation #
Implementation details #
This file should avoid depending on other parts of GroupTheory
, to avoid import cycles.
More sophisticated lemmas belong in GroupTheory.GroupAction
.
Tags #
group action
Embedding of α
into functions M → α
induced by a multiplicative action of M
on α
.
Equations
- MulAction.toFun M α = { toFun := fun (y : α) (x : M) => x • y, inj' := ⋯ }
Instances For
Embedding of α
into functions M → α
induced by an additive action of M
on α
.
Equations
- AddAction.toFun M α = { toFun := fun (y : α) (x : M) => x +ᵥ y, inj' := ⋯ }
Instances For
The monoid of endomorphisms.
Note that this is generalized by CategoryTheory.End
to categories other than Type u
.
Equations
- Function.End α = (α → α)
Instances For
Equations
- instMonoidEnd = Monoid.mk ⋯ ⋯ (fun (n : ℕ) (f : Function.End α) => f^[n]) ⋯ ⋯
Equations
- instInhabitedEnd = { default := 1 }
The tautological action by Function.End α
on α
.
This is generalized to bundled endomorphisms by:
Equiv.Perm.applyMulAction
AddMonoid.End.applyDistribMulAction
AddMonoid.End.applyModule
AddAut.applyDistribMulAction
MulAut.applyMulDistribMulAction
LinearEquiv.applyDistribMulAction
LinearMap.applyModule
RingHom.applyMulSemiringAction
RingAut.applyMulSemiringAction
AlgEquiv.applyMulSemiringAction
Equations
Function.End.applyMulAction
is faithful.
The monoid hom representing a monoid action.
When M
is a group, see MulAction.toPermHom
.
Equations
- MulAction.toEndHom = { toFun := fun (x1 : M) (x2 : α) => x1 • x2, map_one' := ⋯, map_mul' := ⋯ }
Instances For
The additive monoid hom representing an additive monoid action.
When M
is a group, see AddAction.toPermHom
.
Instances For
The monoid action induced by a monoid hom to Function.End α
See note [reducible non-instances].
Equations
Instances For
The additive action induced by a hom to Additive (Function.End α)
See note [reducible non-instances].