Documentation

Mathlib.CategoryTheory.Monoidal.Internal.FunctorCategory

Mon (C ⥤ D) ≌ C ⥤ Mon D #

When D is a monoidal category, monoid objects in C ⥤ D are the same thing as functors from C into the monoid objects of D.

This is formalised as:

The intended application is that as Ring ≌ Mon Ab (not yet constructed!), we have presheaf Ring X ≌ presheaf (Mon Ab) X ≌ Mon (presheaf Ab X), and we can model a module over a presheaf of rings as a module object in presheaf Ab X.

Future work #

Presumably this statement is not specific to monoids, and could be generalised to any internal algebraic objects, if the appropriate framework was available.

A monoid object in a functor category sends any object to a monoid object.

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

    A monoid object in a functor category induces a functor to the category of monoid objects.

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

      Functor translating a monoid object in a functor category to a functor into the category of monoid objects.

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

        A functor to the category of monoid objects can be translated as a monoid object in the functor category.

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

          Functor translating a functor into the category of monoid objects to a monoid object in the functor category

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[simp]
            theorem CategoryTheory.Monoidal.MonFunctorCategoryEquivalence.inverse_map_hom_app {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] {X✝ Y✝ : Functor C (Mon D)} (α : X✝ Y✝) (X : C) :
            (inverse.map α).hom.app X = (α.app X).hom

            The unit for the equivalence Mon (C ⥤ D) ≌ C ⥤ Mon D.

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

              The counit for the equivalence Mon (C ⥤ D) ≌ C ⥤ Mon D.

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

                When D is a monoidal category, monoid objects in C ⥤ D are the same thing as functors from C into the monoid objects of D.

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

                  A comonoid object in a functor category sends any object to a comonoid object.

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

                    A comonoid object in a functor category induces a functor to the category of comonoid objects.

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

                      Functor translating a comonoid object in a functor category to a functor into the category of comonoid objects.

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

                        A functor to the category of comonoid objects can be translated as a comonoid object in the functor category.

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

                          The counit for the equivalence Mon (C ⥤ D) ≌ C ⥤ Mon D.

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

                            When D is a monoidal category, comonoid objects in C ⥤ D are the same thing as functors from C into the comonoid objects of D.

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

                              Functor translating a commutative monoid object in a functor category to a functor into the category of commutative monoid objects.

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

                                Functor translating a functor into the category of commutative monoid objects to a commutative monoid object in the functor category

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

                                  The unit for the equivalence CommMon (C ⥤ D) ≌ C ⥤ CommMon D.

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

                                    The counit for the equivalence CommMon (C ⥤ D) ≌ C ⥤ CommMon D.

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

                                      When D is a braided monoidal category, commutative monoid objects in C ⥤ D are the same thing as functors from C into the commutative monoid objects of D.

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