Internal homs for day convolution #
Given a category V
that is monoidal closed, a category C
that
is monoidal, a functor C ⥤ V
, and given the data of suitable day convolutions
and suitable ends of profunctors c c₁ c₂ ↦ ihom (F c₁) (·.obj (c₂ ⊗ c))
,
we prove that the data of the units of the left Kan extensions that define
day convolutions and the data of the canonical morphisms to the aforementioned
ends can be organised as data that exhibit F
as monoidal closed in C ⥤ V
for
the Day convolution monoidal structure.
TODOs #
- When
LawfulDayConvolutionMonoidalStruct
(#26820) lands, transport the constructions here to produce actualCategoryTheory.MonoidalClosed
instances.
Given F : C ⥤ V
, this is the functor
G ↦ c c₁ c₂ ↦ ihom (F c₁) (G.obj (c₂ ⊗ c))
.
The internal hom functor for Day convolution [F, -]
is naturally isomorphic
to the functor G ↦ c ↦ end_ (c₁ c₂ ↦ ihom (F c₁) (G.obj (c₂ ⊗ c)))
, hence
this definition.
Equations
- One or more equations did not get rendered due to their size.
Instances For
DayConvolutionInternalHom F G H
asserts that H
is the value at G
of
an internal hom functor of F
for the Day convolution monoidal structure.
This is phrased as the data of a limit CategoryTheory.Wedge
(i.e an end) on internalHomDiagramFunctor F|>.obj G|>.obj c
and
c
, with tip (H.obj G).obj c
and a compatibility condition asserting that
the functoriality of H
identifies to the functoriality of ends.
The canonical projections maps
- hπ (c : C) ⦃i j : C⦄ (f : i ⟶ j) : CategoryStruct.comp (self.π c i) ((ihom (F.obj i)).map (G.map (whiskerRight f c))) = CategoryStruct.comp (self.π c j) ((MonoidalClosed.pre (F.map f)).app (G.obj (tensorObj j c)))
The projections maps assemble into a wedge.
- isLimitWedge (c : C) : Limits.IsLimit (Limits.Wedge.mk (H.obj c) (self.π c) ⋯)
- map_comp_π {c c' : C} (f : c ⟶ c') (j : C) : CategoryStruct.comp (H.map f) (self.π c' j) = CategoryStruct.comp (self.π c j) ((ihom (F.obj j)).map (G.map (whiskerLeft j f)))
The functoriality of
H.obj G
identifies (throughWedge.IsLimit.hom_ext
) with the functoriality on ends induced by functoriality ofinternalHomDiagramFunctor F|>.obj G
.
Instances For
If we have a map G ⟶ G'
and a DayConvolutionInternalHom F G' H'
, then
there is a unique map H ⟶ H'
induced by functoriality of ends and functoriality
of internalHomDiagramFunctor F
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given ℌ : DayConvolutionInternalHom F H
, if we think of H.obj G
as the internal hom [F, G]
, then this is the transformation
corresponding to the component at G
of the "evaluation" natural morphism
F ⊛ [F, _] ⟶ 𝟭
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given ℌ : DayConvolutionInternalHom F H
, if we think of H.obj G
as the internal hom [F, G]
, then this is the transformation
corresponding to the component at G
of the "coevaluation" natural morphism
𝟭 ⟶ [F, F ⊛ _]
.
Equations
- One or more equations did not get rendered due to their size.