The Coherent Grothendieck Topology #
This file defines the coherent Grothendieck topology (and coverage) on a category C
.
The category C
must satisfy a Precoherent C
condition, which is essentially the minimal
requirement for the coherent coverage to exist.
Given such a category, the coherent coverage is coherentCoverage C
and the corresponding
Grothendieck topology is coherentTopology C
.
In isSheaf_coherent
, we characterize the sheaf condition for presheaves of types for the
coherent Grothendieck topology in terms of finite effective epimorphic families.
References: #
- [Elephant]: Sketches of an Elephant, P. T. Johnstone: C2.1, Example 2.1.12.
- nLab, Coherent Coverage
- pullback : ∀ {B₁ B₂ : C} (f : B₂ ⟶ B₁) (α : Type) [inst : Fintype α] (X₁ : α → C) (π₁ : (a : α) → X₁ a ⟶ B₁), CategoryTheory.EffectiveEpiFamily X₁ π₁ → ∃ β x X₂ π₂, CategoryTheory.EffectiveEpiFamily X₂ π₂ ∧ ∃ i ι, ∀ (b : β), CategoryTheory.CategoryStruct.comp (ι b) (π₁ (i b)) = CategoryTheory.CategoryStruct.comp (π₂ b) f
Given an effective epi family
π₁
overB₁
and a morphismf : B₂ ⟶ B₁
, there exists an effective epi familyπ₂
overB₂
, such thatπ₂
factors throughπ₁
.
The condition Precoherent C
is essentially the minimal condition required to define the
coherent coverage on C
.
Instances
The coherent coverage on a precoherent category C
.
Instances For
The coherent Grothendieck topology on a precoherent category C
.
Instances For
For a precoherent category, any sieve that contains an EffectiveEpiFamily
is a sieve of the
coherent topology.
Note: This is one direction of mem_sieves_iff_hasEffectiveEpiFamily
, but is needed for the proof.
Every Yoneda-presheaf is a sheaf for the coherent topology.
The coherent topology on a precoherent category is subcanonical.
Effective epi families in a precoherent category are transitive, in the sense that an
EffectiveEpiFamily
and an EffectiveEpiFamily
over each member, the composition is an
EffectiveEpiFamily
.
Note: The finiteness condition is an artifact of the proof and is probably unnecessary.
A sieve belongs to the coherent topology if and only if it contains a finite
EffectiveEpiFamily
.