Documentation

Mathlib.CategoryTheory.Sites.Sheafification

Sheafification #

We construct the sheafification of a presheaf over a site C with values in D whenever D is a concrete category for which the forgetful functor preserves the appropriate (co)limits and reflects isomorphisms.

We generally follow the approach of https://stacks.math.columbia.edu/tag/00W1

A concrete version of the multiequalizer, to be used below.

Instances For
    def CategoryTheory.GrothendieckTopology.Plus.meqOfSep {C : Type u} [CategoryTheory.Category.{v, u} C] {J : CategoryTheory.GrothendieckTopology C} {D : Type w} [CategoryTheory.Category.{max v u, w} D] [CategoryTheory.ConcreteCategory D] [CategoryTheory.Limits.PreservesLimits (CategoryTheory.forget D)] [∀ (X : C), CategoryTheory.Limits.HasColimitsOfShape (CategoryTheory.GrothendieckTopology.Cover J X)ᵒᵖ D] [∀ (P : CategoryTheory.Functor Cᵒᵖ D) (X : C) (S : CategoryTheory.GrothendieckTopology.Cover J X), CategoryTheory.Limits.HasMultiequalizer (CategoryTheory.GrothendieckTopology.Cover.index S P)] [(X : C) → CategoryTheory.Limits.PreservesColimitsOfShape (CategoryTheory.GrothendieckTopology.Cover J X)ᵒᵖ (CategoryTheory.forget D)] (P : CategoryTheory.Functor Cᵒᵖ D) (hsep : ∀ (X : C) (S : CategoryTheory.GrothendieckTopology.Cover J X) (x y : (CategoryTheory.forget D).obj (P.obj (Opposite.op X))), (∀ (I : CategoryTheory.GrothendieckTopology.Cover.Arrow S), ↑(P.map I.f.op) x = ↑(P.map I.f.op) y) → x = y) (X : C) (S : CategoryTheory.GrothendieckTopology.Cover J X) (s : CategoryTheory.Meq (CategoryTheory.GrothendieckTopology.plusObj J P) S) (T : (I : CategoryTheory.GrothendieckTopology.Cover.Arrow S) → CategoryTheory.GrothendieckTopology.Cover J I.Y) (t : (I : CategoryTheory.GrothendieckTopology.Cover.Arrow S) → CategoryTheory.Meq P (T I)) (ht : ∀ (I : CategoryTheory.GrothendieckTopology.Cover.Arrow S), s I = CategoryTheory.GrothendieckTopology.Plus.mk (t I)) :

    An auxiliary definition to be used in the proof of exists_of_sep below. Given a compatible family of local sections for P⁺, and representatives of said sections, construct a compatible family of local sections of P over the combination of the covers associated to the representatives. The separatedness condition is used to prove compatibility among these local sections of P.

    Instances For