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 RingMon_ 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 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]
    theorem CategoryTheory.Monoidal.MonFunctorCategoryEquivalence.functorObj_map_hom {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] (A : Mon_ (Functor C D)) {X✝ Y✝ : C} (f : X✝ Y✝) :
    ((functorObj A).map f).hom = A.X.map f

    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]
      theorem CategoryTheory.Monoidal.MonFunctorCategoryEquivalence.functor_map_app_hom {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] {X✝ Y✝ : Mon_ (Functor C D)} (f : X✝ Y✝) (X : C) :
      ((functor.map f).app X).hom = f.hom.app X

      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
            @[simp]
            @[simp]

            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
              @[simp]
              @[simp]

              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 induces a functor to the category of comonoid objects.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[simp]
                  theorem CategoryTheory.Monoidal.ComonFunctorCategoryEquivalence.functorObj_map_hom {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] (A : Comon_ (Functor C D)) {X✝ Y✝ : C} (f : X✝ Y✝) :
                  ((functorObj A).map f).hom = A.X.map f

                  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
                    @[simp]
                    theorem CategoryTheory.Monoidal.ComonFunctorCategoryEquivalence.functor_map_app_hom {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] {X✝ Y✝ : Comon_ (Functor C D)} (f : X✝ Y✝) (X : C) :
                    ((functor.map f).app X).hom = f.hom.app X

                    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
                            @[simp]
                            theorem CategoryTheory.Monoidal.CommMonFunctorCategoryEquivalence.functor_map_app_hom {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] [BraidedCategory D] {X✝ Y✝ : CommMon_ (Functor C D)} (f : X✝ Y✝) (X : C) :
                            ((functor.map f).app X).hom = f.hom.app X
                            @[simp]
                            theorem CategoryTheory.Monoidal.CommMonFunctorCategoryEquivalence.functor_obj_map_hom {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] [BraidedCategory D] (A : CommMon_ (Functor C D)) {X Y : C} (a✝ : X Y) :
                            ((functor.obj A).map a✝).hom = A.X.map a✝

                            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
                              @[simp]
                              theorem CategoryTheory.Monoidal.CommMonFunctorCategoryEquivalence.inverse_obj_X_map {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] [BraidedCategory D] (F : Functor C (CommMon_ D)) {X✝ Y✝ : C} (f : X✝ Y✝) :
                              (inverse.obj F).X.map f = (F.map f).hom
                              @[simp]
                              theorem CategoryTheory.Monoidal.CommMonFunctorCategoryEquivalence.inverse_map_hom_app {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] [MonoidalCategory D] [BraidedCategory D] {X✝ Y✝ : Functor C (CommMon_ D)} (α : X✝ Y✝) (X : C) :
                              (inverse.map α).hom.app X = (α.app X).hom

                              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