Documentation

Mathlib.CategoryTheory.Sites.Sheafification

Sheafification #

Given a site (C, J) we define a typeclass HasSheafify J A saying that the inclusion functor from A-valued sheaves on C to presheaves admits a left exact left adjoint (sheafification).

Note: to access the HasSheafify instance for suitable concrete categories, import the file Mathlib.CategoryTheory.Sites.LeftExact.

@[reducible, inline]

A proposition saying that the inclusion functor from sheaves to presheaves admits a left adjoint.

Equations
Instances For

    HasSheafify means that the inclusion functor from sheaves to presheaves admits a left exact left adjiont (sheafification).

    Given a finite limit preserving functor F : (Cᵒᵖ ⥤ A) ⥤ Sheaf J A and an adjunction adj : F ⊣ sheafToPresheaf J A, use HasSheafify.mk' to construct a HasSheafify instance.

    Instances

      The sheafification functor, left adjoint to the inclusion.

      Equations
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        @[reducible, inline]

        The sheafification of a presheaf P.

        Equations
        Instances For
          @[reducible, inline]
          noncomputable abbrev CategoryTheory.toSheafify {C : Type u₁} [Category.{v₁, u₁} C] (J : GrothendieckTopology C) {D : Type u_1} [Category.{u_2, u_1} D] [HasWeakSheafify J D] (P : Functor Cᵒᵖ D) :

          The canonical map from P to its sheafification.

          Equations
          Instances For
            @[reducible, inline]
            noncomputable abbrev CategoryTheory.sheafifyMap {C : Type u₁} [Category.{v₁, u₁} C] (J : GrothendieckTopology C) {D : Type u_1} [Category.{u_2, u_1} D] [HasWeakSheafify J D] {P Q : Functor Cᵒᵖ D} (η : P Q) :

            The canonical map on sheafifications induced by a morphism.

            Equations
            Instances For
              @[reducible, inline]

              The sheafification of a presheaf P, as a functor.

              Equations
              Instances For
                @[reducible, inline]

                The canonical map from P to its sheafification, as a natural transformation.

                Equations
                Instances For

                  If P is a sheaf, then P is isomorphic to sheafify J P.

                  Equations
                  Instances For
                    noncomputable def CategoryTheory.sheafifyLift {C : Type u₁} [Category.{v₁, u₁} C] (J : GrothendieckTopology C) {D : Type u_1} [Category.{u_2, u_1} D] [HasWeakSheafify J D] {P Q : Functor Cᵒᵖ D} (η : P Q) (hQ : Presheaf.IsSheaf J Q) :

                    Given a sheaf Q and a morphism P ⟶ Q, construct a morphism from sheafify J P to Q.

                    Equations
                    Instances For
                      theorem CategoryTheory.sheafifyLift_unique {C : Type u₁} [Category.{v₁, u₁} C] (J : GrothendieckTopology C) {D : Type u_1} [Category.{u_2, u_1} D] [HasWeakSheafify J D] {P Q : Functor Cᵒᵖ D} (η : P Q) (hQ : Presheaf.IsSheaf J Q) (γ : sheafify J P Q) :
                      CategoryStruct.comp (toSheafify J P) γ = ηγ = sheafifyLift J η hQ
                      noncomputable def CategoryTheory.sheafificationIso {C : Type u₁} [Category.{v₁, u₁} C] {J : GrothendieckTopology C} {D : Type u_1} [Category.{u_2, u_1} D] [HasWeakSheafify J D] (P : Sheaf J D) :
                      P (presheafToSheaf J D).obj P.val

                      A sheaf P is isomorphic to its own sheafification.

                      Equations
                      Instances For

                        The natural isomorphism 𝟭 (Sheaf J D) ≅ sheafToPresheaf J D ⋙ presheafToSheaf J D.

                        Equations
                        Instances For