Documentation

Mathlib.CategoryTheory.Sites.Grothendieck

Grothendieck topologies #

Definition and lemmas about Grothendieck topologies. A Grothendieck topology for a category C is a set of sieves on each object X satisfying certain closure conditions.

Alternate versions of the axioms (in arrow form) are also described. Two explicit examples of Grothendieck topologies are given:

A pretopology, or a basis for a topology is defined in Mathlib/CategoryTheory/Sites/Pretopology.lean. The topology associated to a topological space is defined in Mathlib/CategoryTheory/Sites/Spaces.lean.

Tags #

Grothendieck topology, coverage, pretopology, site

References #

Implementation notes #

We use the definition of [nlab] and [MM92][] (Chapter III, Section 2), where Grothendieck topologies are saturated collections of morphisms, rather than the notions of the Stacks project (00VG) and the Elephant, in which topologies are allowed to be unsaturated, and are then completed. TODO (BM): Add the definition from Stacks, as a pretopology, and complete to a topology.

This is so that we can produce a bijective correspondence between Grothendieck topologies on a small category and Lawvere-Tierney topologies on its presheaf topos, as well as the equivalence between Grothendieck topoi and left exact reflective subcategories of presheaf toposes.

The definition of a Grothendieck topology: a set of sieves J X on each object X satisfying three axioms:

  1. For every object X, the maximal sieve is in J X.
  2. If S ∈ J X then its pullback along any h : Y ⟶ X is in J Y.
  3. If S ∈ J X and R is a sieve on X, then provided that the pullback of R along any arrow f : Y ⟶ X in S is in J Y, we have that R itself is in J X.

A sieve S on X is referred to as J-covering, (or just covering), if S ∈ J X.

See , or [nlab], or [MM92][] Chapter III, Section 2, Definition 1.

Instances For

    An extensionality lemma in terms of the coercion to a pi-type. We prove this explicitly rather than deriving it so that it is in terms of the coercion rather than the projection .sieves.

    @[simp]

    Also known as the maximality axiom.

    @[simp]

    Also known as the stability axiom.

    theorem CategoryTheory.GrothendieckTopology.transitive {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {S : CategoryTheory.Sieve X} (J : CategoryTheory.GrothendieckTopology C) (hS : S J.sieves X) (R : CategoryTheory.Sieve X) (h : ∀ ⦃Y : C⦄ ⦃f : Y X⦄, S.arrows fCategoryTheory.Sieve.pullback f R J.sieves Y) :
    R J.sieves X

    If S is a subset of R, and S is covering, then R is covering as well.

    See (2), or discussion after [MM92] Chapter III, Section 2, Definition 1.

    The intersection of two covering sieves is covering.

    See (1), or [MM92] Chapter III, Section 2, Definition 1 (iv).

    theorem CategoryTheory.GrothendieckTopology.bind_covering {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} (J : CategoryTheory.GrothendieckTopology C) {S : CategoryTheory.Sieve X} {R : Y : C⦄ → f : Y X⦄ → S.arrows fCategoryTheory.Sieve Y} (hS : S J.sieves X) (hR : ∀ ⦃Y : C⦄ ⦃f : Y X⦄ (H : S.arrows f), R H J.sieves Y) :
    CategoryTheory.Sieve.bind S.arrows R J.sieves X

    The sieve S on X J-covers an arrow f to X if S.pullback f ∈ J Y. This definition is an alternate way of presenting a Grothendieck topology.

    Equations
    Instances For

      The maximality axiom in 'arrow' form: Any arrow f in S is covered by S.

      The stability axiom in 'arrow' form: If S covers f then S covers g ≫ f for any g.

      The transitivity axiom in 'arrow' form: If S covers f and every arrow in S is covered by R, then R covers f.

      The trivial Grothendieck topology, in which only the maximal sieve is covering. This topology is also known as the indiscrete, coarse, or chaotic topology.

      See [MM92] Chapter III, Section 2, example (a), or https://en.wikipedia.org/wiki/Grothendieck_topology#The_discrete_and_indiscrete_topologies

      Equations
      Instances For

        The discrete Grothendieck topology, in which every sieve is covering.

        See https://en.wikipedia.org/wiki/Grothendieck_topology#The_discrete_and_indiscrete_topologies.

        Equations
        Instances For

          See

          Equations

          See

          Equations
          • CategoryTheory.GrothendieckTopology.instPartialOrderGrothendieckTopology = let __src := CategoryTheory.GrothendieckTopology.instLEGrothendieckTopology; PartialOrder.mk

          See

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

          Construct a complete lattice from the Inf, but make the trivial and discrete topologies definitionally equal to the bottom and top respectively.

          Equations
          • One or more equations did not get rendered due to their size.
          Equations
          • CategoryTheory.GrothendieckTopology.instInhabitedGrothendieckTopology = { default := }

          The dense Grothendieck topology.

          See https://ncatlab.org/nlab/show/dense+topology, or [MM92] Chapter III, Section 2, example (e).

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem CategoryTheory.GrothendieckTopology.dense_covering {C : Type u} [CategoryTheory.Category.{v, u} C] {X : C} {S : CategoryTheory.Sieve X} :
            S CategoryTheory.GrothendieckTopology.dense.sieves X ∀ {Y : C} (f : Y X), ∃ (Z : C) (g : Z Y), S.arrows (CategoryTheory.CategoryStruct.comp g f)

            A category satisfies the right Ore condition if any span can be completed to a commutative square. NB. Any category with pullbacks obviously satisfies the right Ore condition, see right_ore_of_pullbacks.

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

              The atomic Grothendieck topology: a sieve is covering iff it is nonempty. For the pullback stability condition, we need the right Ore condition to hold.

              See https://ncatlab.org/nlab/show/atomic+site, or [MM92] Chapter III, Section 2, example (f).

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

                J.Cover X denotes the poset of covers of X with respect to the Grothendieck topology J.

                Equations
                Instances For
                  Equations
                  • CategoryTheory.GrothendieckTopology.Cover.instOrderTopCoverToLEInstPreorderCover = let __src := inferInstance; OrderTop.mk
                  Equations
                  • CategoryTheory.GrothendieckTopology.Cover.instSemilatticeInfCover = let __src := inferInstance; SemilatticeInf.mk
                  Equations
                  • CategoryTheory.GrothendieckTopology.Cover.instInhabitedCover = { default := }

                  An auxiliary structure, used to define S.index.

                  Instances For
                    theorem CategoryTheory.GrothendieckTopology.Cover.Relation.ext_iff {C : Type u} :
                    ∀ {inst : CategoryTheory.Category.{v, u} C} {X : C} {J : CategoryTheory.GrothendieckTopology C} {S : CategoryTheory.GrothendieckTopology.Cover J X} (x y : CategoryTheory.GrothendieckTopology.Cover.Relation S), x = y x.Y₁ = y.Y₁ x.Y₂ = y.Y₂ x.Z = y.Z HEq x.g₁ y.g₁ HEq x.g₂ y.g₂ HEq x.f₁ y.f₁ HEq x.f₂ y.f₂
                    theorem CategoryTheory.GrothendieckTopology.Cover.Relation.ext {C : Type u} :
                    ∀ {inst : CategoryTheory.Category.{v, u} C} {X : C} {J : CategoryTheory.GrothendieckTopology C} {S : CategoryTheory.GrothendieckTopology.Cover J X} (x y : CategoryTheory.GrothendieckTopology.Cover.Relation S), x.Y₁ = y.Y₁x.Y₂ = y.Y₂x.Z = y.ZHEq x.g₁ y.g₁HEq x.g₂ y.g₂HEq x.f₁ y.f₁HEq x.f₂ y.f₂x = y

                    An auxiliary structure, used to define S.index.

                    Instances For

                      Map a Relation along a refinement S ⟶ T.

                      Equations
                      Instances For

                        Combine a family of covers over a cover.

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

                          An arrow in bind has the form A ⟶ B ⟶ X where A ⟶ B is an arrow in T I for some I. and B ⟶ X is an arrow of S. This is the hom B ⟶ X, as an arrow.

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

                            To every S : J.Cover X and presheaf P, associate a MulticospanIndex.

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

                              The natural multifork associated to S : J.Cover X for a presheaf P. Saying that this multifork is a limit is essentially equivalent to the sheaf condition at the given object for the given covering sieve. See Sheaf.lean for an equivalent sheaf condition using this.

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

                                The canonical map from P.obj (op X) to the multiequalizer associated to a covering sieve, assuming such a multiequalizer exists. This will be used in Sheaf.lean to provide an equivalent sheaf condition in terms of multiequalizers.

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

                                  Pull back a cover along a morphism.

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

                                    Pulling back along the identity is naturally isomorphic to the identity functor.

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

                                      Pulling back along a composition is naturally isomorphic to the composition of the pullbacks.

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