Existence of conical limits #
This file contains different statements about the (non-constructive) existence of conical limits.
The main constructions are the following.
HasConicalLimit
: there exists a conical limit forF : J ⥤ C
.HasConicalLimitsOfShape J
: All functorsF : J ⥤ C
have conical limits.HasConicalLimitsOfSize.{v₁, u₁}
: For all smallJ
all functorsF : J ⥤ C
have conical limits.HasConicalLimits
:C
has all (small) conical limits.
References #
- Kelly G.M., Basic concepts of enriched category theory: See section 3.8 for a similar treatment, although the content of this file is not directly adapted from there.
Implementation notes #
V
has been made an (V : outParam <| Type u')
in the classes below as it seems instance
inference prefers this. Otherwise it failed with
cannot find synthesization order
on the instances below.
However, it is not fully clear yet whether this could lead to potential issues, for example
if there are multiple MonoidalCategory _
instances in scope.
HasConicalLimit F
represents the mere existence of a conical limit for F
.
- exists_limit : Nonempty (LimitCone F)
- preservesLimit_eCoyoneda (X : C) : Limits.PreservesLimit F (eCoyoneda V X)
Instances
C
has conical limits of shape J
if there exists a conical limit for every functor F : J ⥤ C
.
- hasConicalLimit (F : Functor J C) : HasConicalLimit V F
All functors
F : J ⥤ C
fromJ
have limits.
Instances
C
has all conical limits of size v₁ u₁
(HasLimitsOfSize.{v₁ u₁} C
)
if it has conical limits of every shape J : Type u₁
with [Category.{v₁} J]
.
All functors
F : J ⥤ C
from all smallJ
have conical limits
Instances
C
has all (small) conical limits if it has limits of every shape that is as big as its
hom-sets.
Equations
Instances For
If a functor F
has a conical limit, so does any naturally isomorphic functor.
If a G ⋙ F
has a limit, and G
is an equivalence, we can construct a limit of F
.
existence of conical limits (of shape) implies existence of limits (of shape)
We can transport conical limits of shape J'
along an equivalence J' ≌ J
.
existence of conical limits (of size) implies existence of limits (of size)