Convolution product on linear maps from a coalgebra to an algebra #
This file constructs the ring structure on linear maps C → A where C is a coalgebra and A an
algebra, where multiplication is given by (f * g)(x) = ∑ f x₍₁₎ * g x₍₂₎ in Sweedler notation or
|
μ
| | / \
f * g = f g
| | \ /
δ
|
diagrammatically, where μ stands for multiplication and δ for comultiplication.
Implementation notes #
Note that in the case C = A this convolution product conflicts with the (unfortunately global!)
group instance on Module.End R A with multiplication defined as composition.
As a result, the convolution product is scoped to ConvolutionProduct.
Convolution product on linear maps from a coalgebra to an algebra.
Equations
- LinearMap.convMul = { mul := fun (f g : C →ₗ[R] A) => LinearMap.mul' R A ∘ₗ TensorProduct.map f g ∘ₗ CoalgebraStruct.comul }
Instances For
Non-unital and non-associative convolution semiring structure on linear maps from a coalgebra to a non-unital non-associative algebra.
Equations
- LinearMap.convNonUnitalNonAssocSemiring = { toAddCommMonoid := LinearMap.addCommMonoid, toMul := LinearMap.convMul, left_distrib := ⋯, right_distrib := ⋯, zero_mul := ⋯, mul_zero := ⋯ }
Instances For
Non-unital and non-associative convolution ring structure on linear maps from a coalgebra to a non-unital and non-associative algebra.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Non-unital convolution semiring structure on linear maps from a coalgebra to a non-unital algebra.
Equations
- LinearMap.convNonUnitalSemiring = { toNonUnitalNonAssocSemiring := LinearMap.convNonUnitalNonAssocSemiring, mul_assoc := ⋯ }
Instances For
Non-unital convolution ring structure on linear maps from a coalgebra to a non-unital algebra.
Equations
- LinearMap.convNonUnitalRing = { toNonUnitalNonAssocRing := LinearMap.convNonUnitalNonAssocRing, mul_assoc := ⋯ }
Instances For
Convolution unit on linear maps from a coalgebra to an algebra.
Equations
- LinearMap.convOne = { one := Algebra.linearMap R A ∘ₗ CoalgebraStruct.counit }
Instances For
Convolution semiring structure on linear maps from a coalgebra to an algebra.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Commutative convolution semiring structure on linear maps from a cocommutative coalgebra to an algebra.
Equations
- LinearMap.convCommSemiring = { toSemiring := LinearMap.convSemiring, mul_comm := ⋯ }
Instances For
Convolution ring structure on linear maps from a coalgebra to an algebra.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Commutative convolution ring structure on linear maps from a cocommutative coalgebra to an algebra.
Equations
- LinearMap.convCommRing = { toRing := LinearMap.convRing, mul_comm := ⋯ }