Sum instances for additive and multiplicative actions #
This file defines instances for additive and multiplicative actions on the binary Sum
type.
See also #
instance
Sum.instIsScalarTowerSumInstSMulSumInstSMulSum
{M : Type u_1}
{N : Type u_2}
{α : Type u_3}
{β : Type u_4}
[inst : SMul M α]
[inst : SMul M β]
[inst : SMul N α]
[inst : SMul N β]
[inst : SMul M N]
[inst : IsScalarTower M N α]
[inst : IsScalarTower M N β]
:
IsScalarTower M N (α ⊕ β)
instance
Sum.instVAddCommClassSumInstVAddSumInstVAddSum
{M : Type u_1}
{N : Type u_2}
{α : Type u_3}
{β : Type u_4}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : VAdd N α]
[inst : VAdd N β]
[inst : VAddCommClass M N α]
[inst : VAddCommClass M N β]
:
VAddCommClass M N (α ⊕ β)
def
Sum.instVAddCommClassSumInstVAddSumInstVAddSum.proof_1
{M : Type u_1}
{N : Type u_2}
{α : Type u_3}
{β : Type u_4}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : VAdd N α]
[inst : VAdd N β]
[inst : VAddCommClass M N α]
[inst : VAddCommClass M N β]
:
VAddCommClass M N (α ⊕ β)
Equations
- (_ : VAddCommClass M N (α ⊕ β)) = (_ : VAddCommClass M N (α ⊕ β))
instance
Sum.instSMulCommClassSumInstSMulSumInstSMulSum
{M : Type u_1}
{N : Type u_2}
{α : Type u_3}
{β : Type u_4}
[inst : SMul M α]
[inst : SMul M β]
[inst : SMul N α]
[inst : SMul N β]
[inst : SMulCommClass M N α]
[inst : SMulCommClass M N β]
:
SMulCommClass M N (α ⊕ β)
def
Sum.instIsCentralVAddSumInstVAddSumAddOpposite.proof_1
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : VAdd Mᵃᵒᵖ α]
[inst : VAdd Mᵃᵒᵖ β]
[inst : IsCentralVAdd M α]
[inst : IsCentralVAdd M β]
:
IsCentralVAdd M (α ⊕ β)
Equations
- (_ : IsCentralVAdd M (α ⊕ β)) = (_ : IsCentralVAdd M (α ⊕ β))
instance
Sum.instIsCentralVAddSumInstVAddSumAddOpposite
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : VAdd Mᵃᵒᵖ α]
[inst : VAdd Mᵃᵒᵖ β]
[inst : IsCentralVAdd M α]
[inst : IsCentralVAdd M β]
:
IsCentralVAdd M (α ⊕ β)
instance
Sum.instIsCentralScalarSumInstSMulSumMulOpposite
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : SMul M α]
[inst : SMul M β]
[inst : SMul Mᵐᵒᵖ α]
[inst : SMul Mᵐᵒᵖ β]
[inst : IsCentralScalar M α]
[inst : IsCentralScalar M β]
:
IsCentralScalar M (α ⊕ β)
def
Sum.FaithfulVAddLeft.proof_1
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : FaithfulVAdd M α]
:
FaithfulVAdd M (α ⊕ β)
Equations
- (_ : FaithfulVAdd M (α ⊕ β)) = (_ : FaithfulVAdd M (α ⊕ β))
instance
Sum.FaithfulVAddLeft
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : FaithfulVAdd M α]
:
FaithfulVAdd M (α ⊕ β)
instance
Sum.FaithfulSMulLeft
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : SMul M α]
[inst : SMul M β]
[inst : FaithfulSMul M α]
:
FaithfulSMul M (α ⊕ β)
instance
Sum.FaithfulVAddRight
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : FaithfulVAdd M β]
:
FaithfulVAdd M (α ⊕ β)
def
Sum.FaithfulVAddRight.proof_1
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : VAdd M α]
[inst : VAdd M β]
[inst : FaithfulVAdd M β]
:
FaithfulVAdd M (α ⊕ β)
Equations
- (_ : FaithfulVAdd M (α ⊕ β)) = (_ : FaithfulVAdd M (α ⊕ β))
instance
Sum.FaithfulSMulRight
{M : Type u_1}
{α : Type u_2}
{β : Type u_3}
[inst : SMul M α]
[inst : SMul M β]
[inst : FaithfulSMul M β]
:
FaithfulSMul M (α ⊕ β)