Documentation

Mathlib.CategoryTheory.Endomorphism

Endomorphisms #

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

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

Endomorphisms of an object in a category. Arguments order in multiplication agrees with Function.comp, not with CategoryTheory.CategoryStruct.comp.

Equations
Instances For

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

    Equations
    Instances For

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

      Equations
      • f.asHom = f
      Instances For

        Endomorphisms of an object form a monoid

        Equations
        • CategoryTheory.End.monoid = Monoid.mk npowRec
        Equations
        Equations

        In a groupoid, endomorphisms form a group

        Equations

        Automorphisms of an object in a category.

        The order of arguments in multiplication agrees with Function.comp, not with CategoryTheory.CategoryStruct.comp.

        Equations
        Instances For
          theorem CategoryTheory.Aut.ext {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {φ₁ : CategoryTheory.Aut X} {φ₂ : CategoryTheory.Aut X} (h : φ₁.hom = φ₂.hom) :
          φ₁ = φ₂

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

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            The inclusion of Aut X to End X as a monoid homomorphism.

            Equations
            Instances For

              Isomorphisms induce isomorphisms of the automorphism group

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                f.map as a monoid hom between endomorphism monoids.

                Equations
                Instances For

                  f.mapIso as a group hom between automorphism groups.

                  Equations
                  Instances For
                    @[simp]
                    theorem CategoryTheory.Functor.mulEquivOfFullyFaithful_symm_apply {C : Type u} [CategoryTheory.Category.{v, u} C] (X : C) {D : Type u'} [CategoryTheory.Category.{v', u'} D] (f : CategoryTheory.Functor C D) [f✝.Full] [f✝.Faithful] (f : f✝.obj X f✝.obj X) :
                    (CategoryTheory.Functor.mulEquivOfFullyFaithful X f✝).symm f = f✝.preimage f

                    equivOfFullyFaithful f as an isomorphism between endomorphism monoids.

                    Equations
                    Instances For
                      @[simp]
                      theorem CategoryTheory.Functor.autMulEquivOfFullyFaithful_symm_apply_inv {C : Type u} [CategoryTheory.Category.{v, u} C] (X : C) {D : Type u'} [CategoryTheory.Category.{v', u'} D] (f : CategoryTheory.Functor C D) [f✝.Full] [f✝.Faithful] (f : f✝.obj X f✝.obj X) :
                      ((CategoryTheory.Functor.autMulEquivOfFullyFaithful X f✝).symm f).inv = f✝.preimage f.inv
                      @[simp]
                      theorem CategoryTheory.Functor.autMulEquivOfFullyFaithful_symm_apply_hom {C : Type u} [CategoryTheory.Category.{v, u} C] (X : C) {D : Type u'} [CategoryTheory.Category.{v', u'} D] (f : CategoryTheory.Functor C D) [f✝.Full] [f✝.Faithful] (f : f✝.obj X f✝.obj X) :
                      ((CategoryTheory.Functor.autMulEquivOfFullyFaithful X f✝).symm f).hom = f✝.preimage f.hom

                      isoEquivOfFullyFaithful f as an isomorphism between automorphism groups.

                      Equations
                      Instances For