Documentation

Mathlib.GroupTheory.GroupAction.SubMulAction.Pointwise

Pointwise monoid structures on SubMulAction #

This file provides SubMulAction.Monoid and weaker typeclasses, which show that SubMulActions inherit the same pointwise multiplications as sets.

To match Submodule.idemSemiring, we do not put these in the Pointwise locale.

def SubMulAction.instOne {R : Type u_1} {M : Type u_2} [Monoid R] [MulAction R M] [One M] :
Equations
Instances For
    theorem SubMulAction.coe_one {R : Type u_1} {M : Type u_2} [Monoid R] [MulAction R M] [One M] :
    Eq (SetLike.coe 1) (Set.range fun (r : R) => HSMul.hSMul r 1)
    theorem SubMulAction.mem_one {R : Type u_1} {M : Type u_2} [Monoid R] [MulAction R M] [One M] {x : M} :
    Iff (Membership.mem 1 x) (Exists fun (r : R) => Eq (HSMul.hSMul r 1) x)
    def SubMulAction.instMul {R : Type u_1} {M : Type u_2} [Monoid R] [MulAction R M] [Mul M] [IsScalarTower R M M] :
    Equations
    Instances For
      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} :
      Iff (Membership.mem (HMul.hMul p q) x) (Exists fun (y : M) => And (Membership.mem p y) (Exists fun (z : M) => And (Membership.mem q z) (Eq (HMul.hMul y z) x)))
      Equations
      Instances For
        def SubMulAction.semiGroup {R : Type u_1} {M : Type u_2} [Monoid R] [MulAction R M] [Semigroup M] [IsScalarTower R M M] :
        Equations
        Instances For
          def 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] :
          Equations
          Instances For
            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 : Nat} :