Presentable objects #
A functor F : C ⥤ D is κ-accessible (Functor.IsCardinalAccessible)
if it commutes with colimits of shape J where J is any κ-filtered category
(that is essentially small relative to the universe w such that κ : Cardinal.{w}.).
We also introduce another typeclass Functor.IsAccessible saying that there exists
a regular cardinal κ such that Functor.IsCardinalAccessible.
An object X of a category is κ-presentable (IsCardinalPresentable)
if the functor Hom(X, _) (i.e. coyoneda.obj (op X)) is κ-accessible.
Similar as for accessible functors, we define a type class IsAccessible.
References #
A functor F : C ⥤ D is κ-accessible (with κ a regular cardinal)
if it preserves colimits of shape J where J is any κ-filtered category.
In the mathematical literature, some assumptions are often made on the
categories C or D (e.g. the existence of κ-filtered colimits,
see HasCardinalFilteredColimits below), but here we do not
make such assumptions.
- preservesColimitOfShape (J : Type w) [SmallCategory J] [IsCardinalFiltered J κ] : Limits.PreservesColimitsOfShape J F
Instances
A functor is accessible relative to a universe w if
it is κ-accessible for some regular κ : Cardinal.{w}.
- exists_cardinal : ∃ (κ : Cardinal.{w}) (x : Fact κ.IsRegular), F.IsCardinalAccessible κ
Instances
An object X in a category is κ-presentable (for κ a regular cardinal)
when the functor Hom(X, _) preserves colimits indexed by
κ-filtered categories.
Equations
Instances For
An object of a category is presentable relative to a universe w
if it is κ-presentable for some regular κ : Cardinal.{w}.
Equations
Instances For
A category has κ-filtered colimits if it has colimits of shape J
for any κ-filtered category J.
- hasColimitsOfShape (J : Type w) [SmallCategory J] [IsCardinalFiltered J κ] : Limits.HasColimitsOfShape J C