(Co)limit presentations #
Let J and C be categories and X : C. We define type ColimitPresentation J X that contains
the data of objects Dⱼ and natural maps sⱼ : Dⱼ ⟶ X that make X the colimit of the Dⱼ.
(See Mathlib/CategoryTheory/Presentable/ColimitPresentation.lean for the construction of a
presentation of a colimit of objects that are equipped with presentations.)
Main definitions: #
CategoryTheory.Limits.ColimitPresentation: A colimit presentation ofXoverJis a diagram{Dᵢ}inCand natural mapssᵢ : Dᵢ ⟶ XmakingXinto the colimit of theDᵢ.CategoryTheory.Limits.LimitPresentation: A limit presentation ofXoverJis a diagram{Dᵢ}inCand natural mapssᵢ : X ⟶ DᵢmakingXinto the limit of theDᵢ.
TODOs: #
- Refactor
TransfiniteCompositionOfShapeso that it extendsColimitPresentation.
A colimit presentation of X over J is a diagram {Dᵢ} in C and natural maps
sᵢ : Dᵢ ⟶ X making X into the colimit of the Dᵢ.
- diag : Functor J C
The diagram
{Dᵢ}. The natural maps
sᵢ : Dᵢ ⟶ X.Xis the colimit of theDᵢviasᵢ.
Instances For
The cocone associated to a colimit presentation.
Instances For
The canonical colimit presentation of any object over a point.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If F : J ⥤ C is a functor that has a colimit, then this is the obvious
colimit presentation of colimit F.
Equations
- CategoryTheory.Limits.ColimitPresentation.colimit F = { diag := F, ι := (CategoryTheory.Limits.getColimitCocone F).1.ι, isColimit := CategoryTheory.Limits.colimit.isColimit F }
Instances For
If F preserves colimits of shape J, it maps colimit presentations of X to
colimit presentations of F(X).
Equations
- One or more equations did not get rendered due to their size.
Instances For
If P is a colimit presentation of X, it is possible to define another
colimit presentation of X where P.diag is replaced by an isomorphic functor.
Equations
- P.changeDiag e = { diag := F, ι := CategoryTheory.CategoryStruct.comp e.hom P.ι, isColimit := (CategoryTheory.Limits.IsColimit.precomposeHomEquiv e { pt := X, ι := P.ι }).invFun P.isColimit }
Instances For
Map a colimit presentation under an isomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Change the index category of a colimit presentation.
Equations
Instances For
A limit presentation of X over J is a diagram {Dᵢ} in C and natural maps
sᵢ : X ⟶ Dᵢ making X into the limit of the Dᵢ.
- diag : Functor J C
The diagram
{Dᵢ}. The natural maps
sᵢ : X ⟶ Dᵢ.Xis the limit of theDᵢviasᵢ.
Instances For
The cone associated to a limit presentation.
Instances For
The canonical limit presentation of any object over a point.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If F : J ⥤ C is a functor that has a limit, then this is the obvious
limit presentation of limit F.
Equations
- CategoryTheory.Limits.LimitPresentation.limit F = { diag := F, π := (CategoryTheory.Limits.getLimitCone F).1.π, isLimit := CategoryTheory.Limits.limit.isLimit F }
Instances For
If F preserves limits of shape J, it maps limit presentations of X to
limit presentations of F(X).
Equations
- One or more equations did not get rendered due to their size.
Instances For
If P is a limit presentation of X, it is possible to define another
limit presentation of X where P.diag is replaced by an isomorphic functor.
Equations
- P.changeDiag e = { diag := F, π := CategoryTheory.CategoryStruct.comp P.π e.inv, isLimit := (CategoryTheory.Limits.IsLimit.postcomposeHomEquiv e.symm { pt := X, π := P.π }).invFun P.isLimit }
Instances For
Map a limit presentation under an isomorphism.
Equations
- P.ofIso e = { diag := P.diag, π := CategoryTheory.CategoryStruct.comp ((CategoryTheory.Functor.const J).map e.inv) P.π, isLimit := P.isLimit.ofIsoLimit (CategoryTheory.Limits.Cones.ext e ⋯) }
Instances For
Change the index category of a limit presentation.