Grothendieck Axioms #
This file defines some of the Grothendieck Axioms for abelian categories, and proves basic facts about them.
Definitions #
HasExactColimitsOfShape J C
-- colimits of shapeJ
inC
are exact.- The dual of the above definitions, called
HasExactLimitsOfShape
. AB4
-- coproducts are exact (this is formulated in terms ofHasExactColimitsOfShape
).AB5
-- filtered colimits are exact (this is formulated in terms ofHasExactColimitsOfShape
).
Theorems #
- The implication from
AB5
toAB4
is established inAB4.ofAB5
. - That
HasExactColimitsOfShape J C
is invariant under equivalences in both parameters is shown inHasExactColimitsOfShape.of_domain_equivalence
andHasExactColimitsOfShape.of_codomain_equivalence
.
Remarks #
For AB4
and AB5
, we only require left exactness as right exactness is automatic.
A comparison with Grothendieck's original formulation of the properties can be found in the
comments of the linked Stacks page.
Exactness as the preservation of short exact sequences is introduced in
CategoryTheory.Abelian.Exact
.
We do not require Abelian
in the definition of AB4
and AB5
because these classes represent
individual axioms. An AB4
category is an abelian category satisfying AB4
, and similarly for
AB5
.
References #
A category C
is said to have exact colimits of shape J
provided that colimits of shape J
exist and are exact (in the sense that they preserve finite limits).
- preservesFiniteLimits : CategoryTheory.Limits.PreservesFiniteLimits CategoryTheory.Limits.colim
Exactness of
J
-shaped colimits stated ascolim : (J ⥤ C) ⥤ C
preserving finite limits.
Instances
A category C
is said to have exact limits of shape J
provided that limits of shape J
exist and are exact (in the sense that they preserve finite colimits).
- preservesFiniteColimits : CategoryTheory.Limits.PreservesFiniteColimits CategoryTheory.Limits.lim
Exactness of
J
-shaped limits stated aslim : (J ⥤ C) ⥤ C
preserving finite colimits.
Instances
Pull back a HasExactColimitsOfShape J
along a functor which preserves and reflects finite limits
and preserves colimits of shape J
Pull back a HasExactLimitsOfShape J
along a functor which preserves and reflects finite colimits
and preserves limits of shape J
Transport a HasExactColimitsOfShape
along an equivalence of the shape.
Note: When C
has finite limits, this lemma holds with the equivalence replaced by a final
functor, see hasExactColimitsOfShape_of_final
below.
Transport a HasExactLimitsOfShape
along an equivalence of the shape.
Note: When C
has finite colimits, this lemma holds with the equivalence replaced by a initial
functor, see hasExactLimitsOfShape_of_initial
below.
A category C
which has coproducts is said to have AB4
of size w
provided that
coproducts of size w
are exact.
- ofShape (α : Type w) : CategoryTheory.HasExactColimitsOfShape (CategoryTheory.Discrete α) C
Instances
A category C
which has coproducts is said to have AB4
provided that
coproducts are exact.
Instances For
A category C
which has products is said to have AB4Star
(in literature AB4*
)
provided that products are exact.
- ofShape (α : Type w) : CategoryTheory.HasExactLimitsOfShape (CategoryTheory.Discrete α) C
Instances
A category C
which has products is said to have AB4Star
(in literature AB4*
)
provided that products are exact.
Instances For
A category C
which has countable coproducts is said to have countable AB4
provided that
countable coproducts are exact.
- ofShape (α : Type) [Countable α] : CategoryTheory.HasExactColimitsOfShape (CategoryTheory.Discrete α) C
Instances
A category C
which has countable coproducts is said to have countable AB4Star
provided that
countable products are exact.
- ofShape (α : Type) [Countable α] : CategoryTheory.HasExactLimitsOfShape (CategoryTheory.Discrete α) C
Instances
A category C
which has filtered colimits of a given size is said to have AB5
of that size
provided that these filtered colimits are exact.
AB5OfSize.{w, w'} C
means that C
has exact colimits of shape J : Type w'
with
Category.{w} J
such that J
is filtered.
- ofShape (J : Type w') [CategoryTheory.Category.{w, w'} J] [CategoryTheory.IsFiltered J] : CategoryTheory.HasExactColimitsOfShape J C
Instances
A category C
which has filtered colimits is said to have AB5
provided that
filtered colimits are exact.
Instances For
A category C
which has cofiltered limits is said to have AB5Star
(in literature AB5*
)
provided that cofiltered limits are exact.
- ofShape (J : Type w') [CategoryTheory.Category.{w, w'} J] [CategoryTheory.IsCofiltered J] : CategoryTheory.HasExactLimitsOfShape J C
Instances
A category C
which has cofiltered limits is said to have AB5Star
(in literature AB5*
)
provided that cofiltered limits are exact.
Instances For
HasExactColimitsOfShape
can be "pushed forward" along final functors
HasExactLimitsOfShape
can be "pushed forward" along initial functors
HasExactColimitsOfShape (Finset (Discrete J)) C
implies HasExactColimitsOfShape (Discrete J) C
A category with finite biproducts and finite limits is AB4 if it is AB5.
A category with finite biproducts and finite limits has countable AB4 if sequential colimits are exact.
HasExactLimitsOfShape (Finset (Discrete J))ᵒᵖ C
implies HasExactLimitsOfShape (Discrete J) C
A category with finite biproducts and finite limits is AB4 if it is AB5.
A category with finite biproducts and finite limits has countable AB4* if sequential limits are exact.
Checking exactness of colimits of shape Discrete ℕ
and Discrete J
for finite J
is enough for
countable AB4.
Checking exactness of limits of shape Discrete ℕ
and Discrete J
for finite J
is enough for
countable AB4*.
Checking AB of shape Discrete ℕ
is enough for countable AB4, provided that the category has
finite biproducts and finite limits.
Checking AB* of shape Discrete ℕ
is enough for countable AB4*, provided that the category has
finite biproducts and finite colimits.
If colim
of shape J
into an abelian category C
preserves monomorphisms, then C
has AB of
shape J
.
If lim
of shape J
into an abelian category C
preserves epimorphisms, then C
has AB* of
shape J
.