Documentation

Mathlib.Algebra.Ring.Action.End

Ring automorphisms #

This file defines the automorphism group structure on RingAut R := RingEquiv R R.

Implementation notes #

The definition of multiplication in the automorphism group agrees with function composition, multiplication in Equiv.Perm, and multiplication in CategoryTheory.End, but not with CategoryTheory.comp.

This file is kept separate from Mathlib/Algebra/Ring/Equiv.lean so that Mathlib.GroupTheory.Perm is free to use equivalences (and other files that use them) before the group structure is defined.

Tags #

ring aut

The tautological action by the group of automorphism of a ring R on R.

Equations
@[simp]
theorem RingAut.smul_def {R : Type u_2} [Semiring R] (f : RingAut R) (r : R) :
f r = f r

Each element of the group defines a ring automorphism.

This is a stronger version of DistribMulAction.toAddAut and MulDistribMulAction.toMulAut.

Equations
Instances For
    @[simp]
    theorem MulSemiringAction.toRingAut_apply (G : Type u_1) (R : Type u_2) [Group G] [Semiring R] [MulSemiringAction G R] (x : G) :
    (toRingAut G R) x = toRingEquiv G R x