Pointwise monoid structures on SubMulAction #
This file provides SubMulAction.Monoid
and weaker typeclasses, which show that SubMulAction
s
inherit the same pointwise multiplications as sets.
To match Submodule.idemSemiring
, we do not put these in the Pointwise
locale.
instance
SubMulAction.instMul
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Mul M]
[IsScalarTower R M M]
:
Mul (SubMulAction R M)
Equations
- SubMulAction.instMul = { mul := fun (p q : SubMulAction R M) => { carrier := Set.image2 (fun (x1 x2 : M) => x1 * x2) ↑p ↑q, smul_mem' := ⋯ } }
theorem
SubMulAction.coe_mul
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Mul M]
[IsScalarTower R M M]
(p q : SubMulAction R M)
:
theorem
SubMulAction.mem_mul
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Mul M]
[IsScalarTower R M M]
{p q : SubMulAction R M}
{x : M}
:
instance
SubMulAction.instMulOneClass
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[MulOneClass M]
[IsScalarTower R M M]
[SMulCommClass R M M]
:
MulOneClass (SubMulAction R M)
Equations
- SubMulAction.instMulOneClass = { one := 1, mul := fun (x1 x2 : SubMulAction R M) => x1 * x2, one_mul := ⋯, mul_one := ⋯ }
@[deprecated SubMulAction.instMulOneClass (since := "04-06-2025")]
def
SubMulAction.mulOneClass
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[MulOneClass M]
[IsScalarTower R M M]
[SMulCommClass R M M]
:
MulOneClass (SubMulAction R M)
Alias of SubMulAction.instMulOneClass
.
Instances For
instance
SubMulAction.instSemigroup
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Semigroup M]
[IsScalarTower R M M]
:
Semigroup (SubMulAction R M)
Equations
- SubMulAction.instSemigroup = { mul := fun (x1 x2 : SubMulAction R M) => x1 * x2, mul_assoc := ⋯ }
@[deprecated SubMulAction.instSemigroup (since := "04-06-2025")]
def
SubMulAction.semiGroup
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Semigroup M]
[IsScalarTower R M M]
:
Semigroup (SubMulAction R M)
Alias of SubMulAction.instSemigroup
.
Equations
Instances For
instance
SubMulAction.instMonoid
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Monoid M]
[IsScalarTower R M M]
[SMulCommClass R M M]
:
Monoid (SubMulAction R M)
Equations
- One or more equations did not get rendered due to their size.
theorem
SubMulAction.coe_pow
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Monoid M]
[IsScalarTower R M M]
[SMulCommClass R M M]
(p : SubMulAction R M)
{n : ℕ}
:
theorem
SubMulAction.subset_coe_pow
{R : Type u_1}
{M : Type u_2}
[Monoid R]
[MulAction R M]
[Monoid M]
[IsScalarTower R M M]
[SMulCommClass R M M]
(p : SubMulAction R M)
{n : ℕ}
: