Documentation

Mathlib.CategoryTheory.Sites.Coherent.RegularTopology

Description of the covering sieves of the regular topology #

This file characterises the covering sieves of the regular topology.

Main result #

theorem CategoryTheory.regularTopology.mem_sieves_of_hasEffectiveEpi {C : Type u_1} [Category.{u_2, u_1} C] [Preregular C] {X : C} (S : Sieve X) :
(∃ (Y : C) (π : Y X), EffectiveEpi π S.arrows π)S (regularTopology C) X

For a preregular category, any sieve that contains an EffectiveEpi is a covering sieve of the regular topology. Note: This is one direction of mem_sieves_iff_hasEffectiveEpi, but is needed for the proof.

Effective epis in a preregular category are stable under composition.

theorem CategoryTheory.regularTopology.mem_sieves_iff_hasEffectiveEpi {C : Type u_1} [Category.{u_2, u_1} C] [Preregular C] {X : C} (S : Sieve X) :
S (regularTopology C) X ∃ (Y : C) (π : Y X), EffectiveEpi π S.arrows π

A sieve is a cover for the regular topology if and only if it contains an EffectiveEpi.