Exactness of colimits #
In this file, we shall study exactness properties of colimits.
First, we translate the assumption that colim : (J ⥤ C) ⥤ C
preserves monomorphisms (resp. preserves epimorphisms, resp. is exact)
into statements involving arbitrary cocones instead of the ones
given by the colimit API. We also show that when an inductive system
involves only monomorphisms, then the "inclusion" morphism
into the colimit is also a monomorphism (assuming J
is filtered and C
satisfies AB5).
Assume that colim : (J ⥤ C) ⥤ C
preserves monomorphisms, and
φ : X₁ ⟶ X₂
is a monomorphism in J ⥤ C
, then if f : c₁.pt ⟶ c₂.pt
is a morphism
between the points of colimit cocones for X₁
and X₂
in such a way that f
idenfities to colim.map φ
, then f
is a monomorphism.
Assume that φ : X₁ ⟶ X₂
is a natural transformation in J ⥤ C
which
consists of epimorphisms, then if f : c₁.pt ⟶ c₂.pt
is a morphism
between the points of cocones c₁
and c₂
for X₁
and X₂
, in such
a way that c₂
is colimit and f
is compatible with φ
, then f
is an epimorphism.
Assume that a functor X : J ⥤ C
maps any morphism to a monomorphism,
that J
is filtered. Then the "inclusion" map c.ι.app j₀
of a colimit cocone for X
is a monomorphism if colim : (Under j₀ ⥤ C) ⥤ C
preserves monomorphisms
(e.g. when C
satisfies AB5).
Given S : ShortCompex (J ⥤ C)
and (colimit) cocones for S.X₁
, S.X₂
,
S.X₃
equipped with suitable data, this is the induced
short complex c₁.pt ⟶ c₂.pt ⟶ c₃.pt
.
Equations
- CategoryTheory.Limits.colim.mapShortComplex S hc₁ c₂ c₃ f g hf hg = CategoryTheory.ShortComplex.mk f g ⋯
Instances For
Assuming HasExactColimitsOfShape J C
, this lemma rephrases the exactness
of the functor colim : (J ⥤ C) ⥤ C
by saying that if S : ShortComplex (J ⥤ C)
is exact, then the short complex obtained by taking the colimits is exact,
where we allow the replacement of the chosen colimit cocones of the
colimit API by arbitrary colimit cocones.