Preservation of (co)limits in the functor category #
- Show that if
X ⨯ -
preserves colimits inD
for anyX : D
, then the product functorF ⨯ -
forF : C ⥤ D
preserves colimits.
The idea of the proof is simply that products and colimits in the functor category are computed pointwise, so pointwise preservation implies general preservation.
- Show that
F ⋙ -
preserves limits if the target category has limits. - Show that
F : C ⥤ D
preserves limits of a certain shape ifLan F.op : Cᵒᵖ ⥤ Type*
preserves such limits.
References #
https://ncatlab.org/nlab/show/commutativity+of+limits+and+colimits#preservation_by_functor_categories_and_localizations
If X × -
preserves colimits in D
for any X : D
, then the product functor F ⨯ -
for
F : C ⥤ D
also preserves colimits.
Note this is (mathematically) a special case of the statement that
"if limits commute with colimits in D
, then they do as well in C ⥤ D
"
but the story in Lean is a bit more complex, and this statement isn't directly a special case.
That is, even with a formalised proof of the general statement, there would still need to be some
work to convert to this version: namely, the natural isomorphism
(evaluation C D).obj k ⋙ prod.functor.obj (F.obj k) ≅ prod.functor.obj F ⋙ (evaluation C D).obj k
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Whiskering right and then taking a limit is the same as taking the limit and applying the functor.
Equations
- CategoryTheory.limitCompWhiskeringRightIsoLimitComp F G = (CategoryTheory.preservesLimitIso ((CategoryTheory.whiskeringRight C D E).obj F) G).symm
Instances For
Equations
- ⋯ = ⋯
Whiskering right and then taking a colimit is the same as taking the colimit and applying the functor.
Equations
- CategoryTheory.colimitCompWhiskeringRightIsoColimitComp F G = (CategoryTheory.preservesColimitIso ((CategoryTheory.whiskeringRight C D E).obj F) G).symm
Instances For
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
If Lan F.op : (Cᵒᵖ ⥤ Type*) ⥤ (Dᵒᵖ ⥤ Type*)
preserves limits of shape J
, so will F
.
F : C ⥤ D ⥤ E
preserves finite limits if it does for each d : D
.
F : C ⥤ D ⥤ E
preserves finite limits if it does for each d : D
.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯