Documentation

Mathlib.CategoryTheory.Sites.Coherent.ExtensiveSheaves

Sheaves for the extensive topology #

This file characterises sheaves for the extensive topology.

Main result #

A presieve is extensive if it is finite and its arrows induce an isomorphism from the coproduct to the target.

Instances
    instance CategoryTheory.instHasPullbacksOfExtensive {C : Type u_1} [Category.{u_3, u_1} C] [FinitaryPreExtensive C] {X : C} (S : Presieve X) [S.Extensive] :
    S.hasPullbacks

    A finite product preserving presheaf is a sheaf for the extensive topology on a category which is FinitaryPreExtensive.

    instance CategoryTheory.instExtensiveOfArrowsι {C : Type u_1} [Category.{u_3, u_1} C] [FinitaryPreExtensive C] {α : Type} [Finite α] (Z : αC) :
    (Presieve.ofArrows Z fun (i : α) => Limits.Sigma.ι Z i).Extensive

    Every Yoneda-presheaf is a sheaf for the extensive topology.

    The extensive topology on a finitary pre-extensive category is subcanonical.

    A presheaf of sets on a category which is FinitaryExtensive is a sheaf iff it preserves finite products.

    A presheaf on a category which is FinitaryExtensive is a sheaf iff it preserves finite products.