Documentation

Mathlib.Algebra.Category.GroupCat.Colimits

The category of additive commutative groups has all colimits. #

This file uses a "pre-automated" approach, just as for Mon/Colimits.lean. It is a very uniform approach, that conceivably could be synthesised directly by a tactic that analyses the shape of AddCommGroup and MonoidHom.

TODO: In fact, in AddCommGroupCat there is a much nicer model of colimits as quotients of finitely supported functions, and we really should implement this as well (or instead).

We build the colimit of a diagram in AddCommGroupCat by constructing the free group on the disjoint union of all the abelian groups in the diagram, then taking the quotient by the abelian group laws within each abelian group, and the identifications given by the morphisms in the diagram.

An inductive type representing all group expressions (without relations) on a collection of types indexed by the objects of J.

Instances For

    The relation on prequotient saying when two expressions are equal because of the abelian group laws, or because one element is mapped to another by a morphism in the diagram.

    Instances For

      The setoid corresponding to group expressions modulo abelian group relations and identifications.

      Equations
      @[simp]
      theorem AddCommGroupCat.Colimits.quot_zero {J : Type u} [CategoryTheory.Category.{v, u} J] (F : CategoryTheory.Functor J AddCommGroupCat) :
      Quot.mk Setoid.r AddCommGroupCat.Colimits.Prequotient.zero = 0

      The function from a given abelian group in the diagram to the colimit abelian group.

      Equations
      Instances For

        The group homomorphism from a given abelian group in the diagram to the colimit abelian group.

        Equations
        Instances For

          The function from the colimit abelian group to the cone point of any other cocone.

          Equations
          Instances For

            The group homomorphism from the colimit abelian group to the cone point of any other cocone.

            Equations
            Instances For

              The categorical cokernel of a morphism in AddCommGroupCat agrees with the usual group-theoretical quotient.

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