Documentation

Mathlib.Algebra.Category.Grp.Colimits

The category of additive commutative groups has all colimits. #

This file constructs colimits in the category of additive commutative groups, as quotients of finitely supported functions.

We build the colimit of a diagram in AddCommGrp 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.

@[reducible, inline]

The relations between elements of the direct sum of the F.obj j given by the morphisms in the diagram J.

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

    The candidate for the colimit of F, defined as the quotient of the direct sum of the commutative groups F.obj j by the relations given by the morphisms in the diagram.

    Equations
    Instances For

      Inclusion of F.obj j into the candidate colimit.

      Equations
      Instances For
        theorem AddCommGrp.Colimits.Quot.addMonoidHom_ext {J : Type u} [CategoryTheory.Category.{v, u} J] (F : CategoryTheory.Functor J AddCommGrp) [DecidableEq J] {α : Type u_1} [AddMonoid α] {f g : Quot F →+ α} (h : ∀ (j : J) (x : (F.obj j)), f ((ι F j) x) = g ((ι F j) x)) :
        f = g

        (implementation detail) Part of the universal property of the colimit cocone, but without assuming that Quot F lives in the correct universe.

        Equations
        Instances For
          @[simp]
          theorem AddCommGrp.Colimits.Quot.ι_desc {J : Type u} [CategoryTheory.Category.{v, u} J] (F : CategoryTheory.Functor J AddCommGrp) (c : CategoryTheory.Limits.Cocone F) [DecidableEq J] (j : J) (x : (F.obj j)) :
          (desc F c) ((ι F j) x) = (c.app j) x
          @[simp]
          theorem AddCommGrp.Colimits.Quot.map_ι {J : Type u} [CategoryTheory.Category.{v, u} J] (F : CategoryTheory.Functor J AddCommGrp) [DecidableEq J] {j j' : J} {f : j j'} (x : (F.obj j)) :
          (ι F j') ((F.map f) x) = (ι F j) x

          (implementation detail) A morphism of commutative additive groups Quot F →+ A induces a cocone on F as long as the universes work out.

          Equations
          Instances For
            @[simp]
            theorem AddCommGrp.Colimits.toCocone_ι_app {J : Type u} [CategoryTheory.Category.{v, u} J] (F : CategoryTheory.Functor J AddCommGrp) [DecidableEq J] {A : Type w} [AddCommGroup A] (f : Quot F →+ A) (j : J) :
            (toCocone F f).app j = f.comp (Quot.ι F j)

            If c is a cocone of F such that Quot.desc F c is bijective, then c is a colimit cocone of F.

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

              (internal implementation) The colimit cocone of a functor F, implemented as a quotient of DFinsupp (fun j ↦ F.obj j), under the assumption that said quotient is small.

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

                If J is w-small, then any functor J ⥤ AddCommGrp.{w} has a colimit.

                @[instance 1300]

                The category of additive commutative groups has all small colimits.

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

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