Functor categories are enriched #
If C
is a V
-enriched ordinary category, then J ⥤ C
is also
a V
-enriched ordinary category, provided C
has suitable limits.
Given two functors F₁
and F₂
from a category J
to a V
-enriched
ordinary category C
, this is the diagram Jᵒᵖ ⥤ J ⥤ V
whose end shall be
the V
-morphisms in J ⥤ V
from F₁
to F₂
.
Equations
- CategoryTheory.Enriched.FunctorCategory.diagram V F₁ F₂ = F₁.op.comp ((CategoryTheory.eHomFunctor V C).comp ((CategoryTheory.whiskeringLeft J C V).obj F₂))
Instances For
The condition that the end diagram V F₁ F₂
exists, see enrichedHom
.
Equations
Instances For
The V
-enriched hom from F₁
to F₂
when F₁
and F₂
are functors J ⥤ C
and C
is a V
-enriched category.
Equations
Instances For
The projection enrichedHom V F₁ F₂ ⟶ F₁.obj j ⟶[V] F₂.obj j
in the category V
for any j : J
when F₁
and F₂
are functors J ⥤ C
and C
is a V
-enriched category.
Equations
Instances For
Given functors F₁
and F₂
in J ⥤ C
, where C
is a V
-enriched ordinary category,
this is the isomorphism (F₁ ⟶ F₂) ≃ (𝟙_ V ⟶ enrichedHom V F₁ F₂)
in the category V
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The identity for the V
-enrichment of the category J ⥤ C
over V
.
Equations
Instances For
The composition for the V
-enrichment of the category J ⥤ C
over V
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If C
is a V
-enriched ordinary category, and C
has suitable limits,
then J ⥤ C
is also a V
-enriched ordinary category.
Equations
- One or more equations did not get rendered due to their size.