Documentation

Mathlib.Algebra.GroupWithZero.Action.End

Group actions and (endo)morphisms #

@[reducible, inline]
abbrev Function.Surjective.distribMulActionLeft {R : Type u_7} {S : Type u_8} {M : Type u_9} [Monoid R] [AddMonoid M] [DistribMulAction R M] [Monoid S] [SMul S M] (f : R →* S) (hf : Function.Surjective f) (hsmul : ∀ (c : R) (x : M), f c x = c x) :

Push forward the action of R on M along a compatible surjective map f : R →* S.

See also Function.Surjective.mulActionLeft and Function.Surjective.moduleLeft.

Equations
Instances For
    @[reducible, inline]
    abbrev DistribMulAction.compHom {M : Type u_1} {N : Type u_2} (A : Type u_3) [AddMonoid A] [Monoid M] [DistribMulAction M A] [Monoid N] (f : N →* M) :

    Compose a DistribMulAction with a MonoidHom, with action f r' • m. See note [reducible non-instances].

    Equations
    Instances For
      @[reducible, inline]
      abbrev MulDistribMulAction.compHom {M : Type u_1} {N : Type u_2} (A : Type u_3) [Monoid A] [Monoid M] [MulDistribMulAction M A] [Monoid N] (f : N →* M) :

      Compose a MulDistribMulAction with a MonoidHom, with action f r' • m. See note [reducible non-instances].

      Equations
      Instances For

        The tautological action by AddMonoid.End α on α.

        This generalizes Function.End.applyMulAction.

        Equations
        @[simp]
        theorem AddMonoid.End.smul_def {α : Type u_5} [AddMonoid α] (f : AddMonoid.End α) (a : α) :
        f a = f a
        def DistribMulAction.toAddEquiv₀ {α : Type u_7} (β : Type u_8) [GroupWithZero α] [AddMonoid β] [DistribMulAction α β] (x : α) (hx : x 0) :
        β ≃+ β

        Each non-zero element of a GroupWithZero defines an additive monoid isomorphism of an AddMonoid on which it acts distributively. This is a stronger version of DistribMulAction.toAddMonoidHom.

        Equations
        Instances For

          Each element of the monoid defines a monoid homomorphism.

          Equations
          Instances For