Functors from a groupoid into a monoidal closed category form a monoidal closed category. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
(Using the pointwise monoidal structure on the functor category.)
Auxiliary definition for category_theory.monoidal_closed.functor_closed
.
The internal hom functor F ⟶[C] -
Equations
Auxiliary definition for category_theory.monoidal_closed.functor_closed
.
The unit for the adjunction (tensor_left F) ⊣ (ihom F)
.
Equations
- F.closed_unit = {app := λ (G : D ⥤ C), {app := λ (X : D), (category_theory.ihom.coev (F.obj X)).app (G.obj X), naturality' := _}, naturality' := _}
Auxiliary definition for category_theory.monoidal_closed.functor_closed
.
The counit for the adjunction (tensor_left F) ⊣ (ihom F)
.
Equations
- F.closed_counit = {app := λ (G : D ⥤ C), {app := λ (X : D), (category_theory.ihom.ev (F.obj X)).app (G.obj X), naturality' := _}, naturality' := _}
If C
is a monoidal closed category and D
is groupoid, then every functor F : D ⥤ C
is
closed in the functor category F : D ⥤ C
with the pointwise monoidal structure.
Equations
- F.closed = {is_adj := {right := F.closed_ihom, adj := category_theory.adjunction.mk_of_unit_counit {unit := F.closed_unit, counit := F.closed_counit, left_triangle' := _, right_triangle' := _}}}
If C
is a monoidal closed category and D
is groupoid, then the functor category D ⥤ C
,
with the pointwise monoidal structure, is monoidal closed.