Documentation

Mathlib.Algebra.Ring.Action.Basic

Group action on rings #

This file defines the typeclass of monoid acting on semirings MulSemiringAction M R, and the corresponding typeclass of invariant subrings.

Note that Algebra does not satisfy the axioms of MulSemiringAction.

Implementation notes #

There is no separate typeclass for group acting on rings, group acting on fields, etc. They are all grouped under MulSemiringAction.

Tags #

group action, invariant subring

class MulSemiringAction (M : Type u) (R : Type v) [Monoid M] [Semiring R] extends DistribMulAction M R :
Type (max u v)

Typeclass for multiplicative actions by monoids on semirings.

This combines DistribMulAction with MulDistribMulAction.

Instances
    @[instance 100]
    instance MulSemiringAction.toMulDistribMulAction (M : Type u_3) (R : Type u_4) {x✝ : Monoid M} {x✝¹ : Semiring R} [h : MulSemiringAction M R] :
    Equations
    def MulSemiringAction.toRingHom (M : Type u_1) [Monoid M] (R : Type v) [Semiring R] [MulSemiringAction M R] (x : M) :
    R →+* R

    Each element of the monoid defines a semiring homomorphism.

    Equations
    Instances For
      @[simp]
      theorem MulSemiringAction.toRingHom_apply (M : Type u_1) [Monoid M] (R : Type v) [Semiring R] [MulSemiringAction M R] (x : M) (x✝ : R) :
      (MulSemiringAction.toRingHom M R x) x✝ = x x✝

      The tautological action by R →+* R on R.

      This generalizes Function.End.applyMulAction.

      Equations
      @[simp]
      theorem RingHom.smul_def (R : Type v) [Semiring R] (f : R →+* R) (a : R) :
      f a = f a

      RingHom.applyMulSemiringAction is faithful.

      Equations
      • =
      @[reducible, inline]
      abbrev MulSemiringAction.compHom {M : Type u_1} {N : Type u_2} [Monoid M] [Monoid N] (R : Type v) [Semiring R] (f : N →* M) [MulSemiringAction M R] :

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

      Equations
      Instances For