Equivariant homomorphisms #
Main definitions #
MulActionHom M X Y
, the type of equivariant functions fromX
toY
, whereM
is a monoid that acts on the typesX
andY
.DistribMulActionHom M A B
, the type of equivariant additive monoid homomorphisms fromA
toB
, whereM
is a monoid that acts on the additive monoidsA
andB
.MulSemiringActionHom M R S
, the type of equivariant ring homomorphisms fromR
toS
, whereM
is a monoid that acts on the ringsR
andS
.
The above types have corresponding classes:
SMulHomClass F M X Y
states thatF
is a type of bundledX → Y→ Y
homs preserving scalar multiplication byM
DistribMulActionHomClass F M A B
states thatF
is a type of bundledA → B→ B
homs preserving the additive monoid structure and scalar multiplication byM
MulSemiringActionHomClass F M R S
states thatF
is a type of bundledR → S→ S
homs preserving the ring structure and scalar multiplication byM
Notations #
X →[M] Y→[M] Y
isMulActionHom M X Y
.A →+[M] B→+[M] B
isDistribMulActionHom M A B
.R →+*[M] S→+*[M] S
isMulSemiringActionHom M R S
.
Equivariant functions.
Equations
- One or more equations did not get rendered due to their size.
The proposition that the function preserves the action.
SMulHomClass F M X Y
states that F
is a type of morphisms preserving
scalar multiplication by M
.
You should extend this class when you extend MulActionHom
.
Instances
Equations
- instSMulHomClassMulActionHom M' X Y = SMulHomClass.mk (_ : ∀ (self : X →[M'] Y) (m : M') (x : X), MulActionHom.toFun self (m • x) = m • MulActionHom.toFun self x)
Turn an element of a type F
satisfying SMulHomClass F M X Y
into an actual
MulActionHom
. This is declared as the default coercion from F
to MulActionHom M X Y
.
Any type satisfying SMulHomClass
can be cast into MulActionHom
via
SMulHomClass.toMulActionHom
.
Equations
- MulActionHom.instCoeTCMulActionHom = { coe := SMulHomClass.toMulActionHom }
The inverse of a bijective equivariant map is equivariant.
Equations
- MulActionHom.inverse f g h₁ h₂ = { toFun := g, map_smul' := (_ : ∀ (m : M) (x : B), g (m • x) = m • g x) }
The proposition that the function preserves 0
map_zero' : MulActionHom.toFun toMulActionHom 0 = 0The proposition that the function preserves addition
map_add' : ∀ (x y : A), MulActionHom.toFun toMulActionHom (x + y) = MulActionHom.toFun toMulActionHom x + MulActionHom.toFun toMulActionHom y
Equivariant additive monoid homomorphisms.
Instances For
Reinterpret an equivariant additive monoid homomorphism as an additive monoid homomorphism.
Equations
- One or more equations did not get rendered due to their size.
Equivariant additive monoid homomorphisms.
Equations
- One or more equations did not get rendered due to their size.
The proposition that the function preserves addition
The proposition that the function preserves 0
map_zero : ∀ (f : F), ↑f 0 = 0
DistribMulActionHomClass F M A B
states that F
is a type of morphisms preserving
the additive monoid structure and scalar multiplication by M
.
You should extend this class when you extend DistribMulActionHom
.
Instances
Equations
- One or more equations did not get rendered due to their size.
Turn an element of a type F
satisfying SMulHomClass F M X Y
into an actual
MulActionHom
. This is declared as the default coercion from F
to MulActionHom M X Y
.
Equations
- One or more equations did not get rendered due to their size.
Any type satisfying SMulHomClass
can be cast into MulActionHom
via
SMulHomClass.toMulActionHom
.
Equations
- DistribMulActionHom.instCoeTCDistribMulActionHom = { coe := DistribMulActionHomClass.toDistribMulActionHom }
The identity map as an equivariant additive monoid homomorphism.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- DistribMulActionHom.instOneDistribMulActionHom = { one := DistribMulActionHom.id M }
Equations
- DistribMulActionHom.instInhabitedDistribMulActionHom = { default := 0 }
Composition of two equivariant additive monoid homomorphisms.
Equations
- One or more equations did not get rendered due to their size.
The inverse of a bijective DistribMulActionHom
is a DistribMulActionHom
.
Equations
- One or more equations did not get rendered due to their size.
The proposition that the function preserves 1
map_one' : MulActionHom.toFun toDistribMulActionHom.toMulActionHom 1 = 1The proposition that the function preserves multiplication
map_mul' : ∀ (x y : R), MulActionHom.toFun toDistribMulActionHom.toMulActionHom (x * y) = MulActionHom.toFun toDistribMulActionHom.toMulActionHom x * MulActionHom.toFun toDistribMulActionHom.toMulActionHom y
Equivariant ring homomorphisms.
Instances For
Reinterpret an equivariant ring homomorphism as a ring homomorphism.
Equations
- One or more equations did not get rendered due to their size.
Equivariant ring homomorphisms.
Equations
- One or more equations did not get rendered due to their size.
The proposition that the function preserves multiplication
The proposition that the function preserves 1
map_one : ∀ (f : F), ↑f 1 = 1
MulSemiringActionHomClass F M R S
states that F
is a type of morphisms preserving
the ring structure and scalar multiplication by M
.
You should extend this class when you extend MulSemiringActionHom
.
Instances
Equations
- One or more equations did not get rendered due to their size.
Turn an element of a type F
satisfying MulSemiringActionHomClass F M R S
into an actual
MulSemiringActionHom
. This is declared as the default coercion from F
to
MulSemiringActionHom M X Y
.
Equations
- One or more equations did not get rendered due to their size.
Any type satisfying MulSemiringActionHomClass
can be cast into MulSemiringActionHom
via
MulSemiringActionHomClass.toMulSemiringActionHom
.
Equations
- MulSemiringActionHom.instCoeTCMulSemiringActionHom = { coe := MulSemiringActionHomClass.toMulSemiringActionHom }
The identity map as an equivariant ring homomorphism.
Equations
- One or more equations did not get rendered due to their size.
Composition of two equivariant additive monoid homomorphisms.
Equations
- One or more equations did not get rendered due to their size.