Documentation

Mathlib.CategoryTheory.Sites.Plus

The plus construction for presheaves. #

This file contains the construction of P⁺, for a presheaf P : Cᵒᵖ ⥤ D where C is endowed with a grothendieck topology J.

See https://stacks.math.columbia.edu/tag/00W1 for details.

The diagram whose colimit defines the values of plus.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.GrothendieckTopology.diagram_map {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] (P : Functor Cᵒᵖ D) (X : C) {S x✝ : (J.Cover X)ᵒᵖ} (f : S x✝) :
    def CategoryTheory.GrothendieckTopology.diagramPullback {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] (P : Functor Cᵒᵖ D) {X Y : C} (f : X Y) :
    J.diagram P Y (J.pullback f).op.comp (J.diagram P X)

    A helper definition used to define the morphisms for plus.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      def CategoryTheory.GrothendieckTopology.diagramNatTrans {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] {P Q : Functor Cᵒᵖ D} (η : P Q) (X : C) :
      J.diagram P X J.diagram Q X

      A natural transformation P ⟶ Q induces a natural transformation between diagrams whose colimits define the values of plus.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        J.diagram P, as a functor in P.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CategoryTheory.GrothendieckTopology.diagramFunctor_map {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) (D : Type w) [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] (X : C) {X✝ Y✝ : Functor Cᵒᵖ D} (η : X✝ Y✝) :

          The plus construction, associating a presheaf to any presheaf. See plusFunctor below for a functorial version.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            An auxiliary definition used in plus below.

            Equations
            Instances For
              @[simp]
              theorem CategoryTheory.GrothendieckTopology.plusMap_comp {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {P Q R : Functor Cᵒᵖ D} (η : P Q) (γ : Q R) :

              The plus construction, a functor sending P to J.plusObj P.

              Equations
              Instances For
                @[simp]
                theorem CategoryTheory.GrothendieckTopology.plusFunctor_map {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) (D : Type w) [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {X✝ Y✝ : Functor Cᵒᵖ D} (η : X✝ Y✝) :
                (J.plusFunctor D).map η = J.plusMap η

                The canonical map from P to J.plusObj P. See toPlusNatTrans for a functorial version.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For

                  The natural transformation from the identity functor to plus.

                  Equations
                  Instances For
                    @[simp]

                    (P ⟶ P⁺)⁺ = P⁺ ⟶ P⁺⁺

                    The natural isomorphism between P and P⁺ when P is a sheaf.

                    Equations
                    Instances For
                      def CategoryTheory.GrothendieckTopology.plusLift {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {P Q : Functor Cᵒᵖ D} (η : P Q) (hQ : Presheaf.IsSheaf J Q) :
                      J.plusObj P Q

                      Lift a morphism P ⟶ Q to P⁺ ⟶ Q when Q is a sheaf.

                      Equations
                      Instances For
                        @[simp]
                        theorem CategoryTheory.GrothendieckTopology.toPlus_plusLift {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {P Q : Functor Cᵒᵖ D} (η : P Q) (hQ : Presheaf.IsSheaf J Q) :
                        theorem CategoryTheory.GrothendieckTopology.plusLift_unique {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {P Q : Functor Cᵒᵖ D} (η : P Q) (hQ : Presheaf.IsSheaf J Q) (γ : J.plusObj P Q) (hγ : CategoryStruct.comp (J.toPlus P) γ = η) :
                        γ = J.plusLift η hQ
                        theorem CategoryTheory.GrothendieckTopology.plus_hom_ext {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {P Q : Functor Cᵒᵖ D} (η γ : J.plusObj P Q) (hQ : Presheaf.IsSheaf J Q) (h : CategoryStruct.comp (J.toPlus P) η = CategoryStruct.comp (J.toPlus P) γ) :
                        η = γ
                        @[simp]
                        theorem CategoryTheory.GrothendieckTopology.plusMap_plusLift {C : Type u} [Category.{v, u} C] (J : GrothendieckTopology C) {D : Type w} [Category.{max v u, w} D] [∀ (P : Functor Cᵒᵖ D) (X : C) (S : J.Cover X), Limits.HasMultiequalizer (S.index P)] [∀ (X : C), Limits.HasColimitsOfShape (J.Cover X)ᵒᵖ D] {P Q R : Functor Cᵒᵖ D} (η : P Q) (γ : Q R) (hR : Presheaf.IsSheaf J R) :