Documentation

Mathlib.Algebra.Category.Grp.FilteredColimits

The forgetful functor from (commutative) (additive) groups preserves filtered colimits. #

Forgetful functors from algebraic categories usually don't preserve colimits. However, they tend to preserve filtered colimits.

In this file, we start with a small filtered category J and a functor F : J ⥤ Grp. We show that the colimit of F ⋙ forget₂ Grp MonCat (in MonCat) carries the structure of a group, thereby showing that the forgetful functor forget₂ Grp MonCat preserves filtered colimits. In particular, this implies that forget Grp preserves filtered colimits. Similarly for AddGrp, CommGrp and AddCommGrp.

@[reducible, inline]

The colimit of F ⋙ forget₂ AddGrp AddMonCat in the category AddMonCat. In the following, we will show that this has the structure of an additive group.

Equations
Instances For
    @[reducible, inline]

    The colimit of F ⋙ forget₂ Grp MonCat in the category MonCat. In the following, we will show that this has the structure of a group.

    Equations
    Instances For
      @[reducible, inline]

      The canonical projection into the colimit, as a quotient type.

      Equations
      Instances For
        @[reducible, inline]

        The canonical projection into the colimit, as a quotient type.

        Equations
        Instances For
          theorem AddGrp.FilteredColimits.G.mk_eq {J : Type v} [CategoryTheory.SmallCategory J] [CategoryTheory.IsFiltered J] (F : CategoryTheory.Functor J AddGrp) (x : (j : J) × (F.obj j)) (y : (j : J) × (F.obj j)) (h : ∃ (k : J) (f : x.fst k) (g : y.fst k), (F.map f) x.snd = (F.map g) y.snd) :
          theorem Grp.FilteredColimits.G.mk_eq {J : Type v} [CategoryTheory.SmallCategory J] [CategoryTheory.IsFiltered J] (F : CategoryTheory.Functor J Grp) (x : (j : J) × (F.obj j)) (y : (j : J) × (F.obj j)) (h : ∃ (k : J) (f : x.fst k) (g : y.fst k), (F.map f) x.snd = (F.map g) y.snd) :

          The "unlifted" version of negation in the colimit.

          Equations
          Instances For

            The "unlifted" version of taking inverses in the colimit.

            Equations
            Instances For
              theorem AddGrp.FilteredColimits.colimitAddGroup.proof_3 {J : Type u_2} [CategoryTheory.SmallCategory J] [CategoryTheory.IsFiltered J] (F : CategoryTheory.Functor J AddGrp) :
              ∀ (n : ) (a : (AddGrp.FilteredColimits.G F)), zsmulRec (↑n.succ) a = zsmulRec (↑n.succ) a

              The bundled additive group giving the filtered colimit of a diagram.

              Equations
              Instances For

                The bundled group giving the filtered colimit of a diagram.

                Equations
                Instances For

                  The cocone over the proposed colimit additive group.

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

                    The cocone over the proposed colimit group.

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

                      The proposed colimit cocone is a colimit in AddGroup.

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

                        The proposed colimit cocone is a colimit in Grp.

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          Equations
                          • One or more equations did not get rendered due to their size.
                          @[reducible, inline]

                          The colimit of F ⋙ forget₂ AddCommGrp AddGrp in the category AddGrp. In the following, we will show that this has the structure of a commutative additive group.

                          Equations
                          Instances For
                            @[reducible, inline]

                            The colimit of F ⋙ forget₂ CommGrp Grp in the category Grp. In the following, we will show that this has the structure of a commutative group.

                            Equations
                            Instances For

                              The bundled additive commutative group giving the filtered colimit of a diagram.

                              Equations
                              Instances For

                                The bundled commutative group giving the filtered colimit of a diagram.

                                Equations
                                Instances For

                                  The cocone over the proposed colimit additive commutative group.

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

                                    The cocone over the proposed colimit commutative group.

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

                                      The proposed colimit cocone is a colimit in AddCommGroup.

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

                                        The proposed colimit cocone is a colimit in CommGrp.

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