mathlib3 documentation

category_theory.endomorphism

Endomorphisms #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Definition and basic properties of endomorphisms and automorphisms of an object in a category.

For each X : C, we provide End X := X ⟶ X with a monoid structure, and Aut X := X ≅ X with a group structure.

@[protected, instance]

Multiplication of endomorphisms agrees with function.comp, not category_struct.comp.

Equations

Assist the typechecker by expressing a morphism X ⟶ X as a term of End X.

Equations

Assist the typechecker by expressing an endomorphism f : End X as a term of X ⟶ X.

Equations
@[simp]
@[simp]
theorem category_theory.End.mul_def {C : Type u} [category_theory.category_struct C] {X : C} (xs ys : category_theory.End X) :
xs * ys = ys xs
@[protected, instance]

Endomorphisms of an object form a monoid

Equations
@[protected, instance]
Equations
theorem category_theory.End.smul_right {C : Type u} [category_theory.category C] {X Y : C} {r : category_theory.End Y} {f : X Y} :
r f = f r
def category_theory.Aut {C : Type u} [category_theory.category C] (X : C) :

Automorphisms of an object in a category.

The order of arguments in multiplication agrees with function.comp, not with category.comp.

Equations
Instances for category_theory.Aut

Units in the monoid of endomorphisms of an object are (multiplicatively) equivalent to automorphisms of that object.

Equations

Isomorphisms induce isomorphisms of the automorphism group

Equations

f.map as a monoid hom between endomorphism monoids.

Equations
@[simp]
theorem category_theory.functor.map_End_apply {C : Type u} [category_theory.category C] (X : C) {D : Type u'} [category_theory.category D] (f : C D) (ᾰ : X X) :

f.map_iso as a group hom between automorphism groups.

Equations