Documentation

Mathlib.CategoryTheory.Sites.Pretopology

Grothendieck pretopologies #

Definition and lemmas about Grothendieck pretopologies. A Grothendieck pretopology for a category C is a set of families of morphisms with fixed codomain, satisfying certain closure conditions.

We show that a pretopology generates a genuine Grothendieck topology, and every topology has a maximal pretopology which generates it.

The pretopology associated to a topological space is defined in Spaces.lean.

Tags #

coverage, pretopology, site

References #

A (Grothendieck) pretopology on C consists of a collection of families of morphisms with a fixed target X for every object X in C, called "coverings" of X, which satisfies the following three axioms:

  1. Every family consisting of a single isomorphism is a covering family.
  2. The collection of covering families is stable under pullback.
  3. Given a covering family, and a covering family on each domain of the former, the composition is a covering family.

In some sense, a pretopology can be seen as Grothendieck topology with weaker saturation conditions, in that each covering is not necessarily downward closed.

See: https://ncatlab.org/nlab/show/Grothendieck+pretopology or [MLM92] Chapter III, Section 2, Definition 2.

Instances For
    theorem CategoryTheory.Pretopology.ext {C : Type u} {inst✝ : Category.{v, u} C} {inst✝¹ : Limits.HasPullbacks C} {x y : Pretopology C} (coverings : x.coverings = y.coverings) :
    x = y
    Equations
    • One or more equations did not get rendered due to their size.
    Equations

    A pretopology K can be completed to a Grothendieck topology J by declaring a sieve to be J-covering if it contains a family in K.

    See also [MLM92] Chapter III, Section 2, Equation (2).

    Equations
    Instances For

      The largest pretopology generating the given Grothendieck topology.

      See [MLM92] Chapter III, Section 2, Equations (3,4).

      Equations
      Instances For
        @[deprecated CategoryTheory.GrothendieckTopology.toPretopology (since := "2025-09-19")]

        Alias of CategoryTheory.GrothendieckTopology.toPretopology.


        The largest pretopology generating the given Grothendieck topology.

        See [MLM92] Chapter III, Section 2, Equations (3,4).

        Equations
        Instances For

          We have a Galois insertion from pretopologies to Grothendieck topologies.

          Equations
          Instances For
            @[deprecated CategoryTheory.GrothendieckTopology.mem_toPretopology (since := "2025-09-19")]

            Alias of CategoryTheory.GrothendieckTopology.mem_toPretopology.

            The trivial pretopology, in which the coverings are exactly singleton isomorphisms. This topology is also known as the indiscrete, coarse, or chaotic topology.

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

              The trivial pretopology induces the trivial Grothendieck topology.

              Equations
              • One or more equations did not get rendered due to their size.
              theorem CategoryTheory.Pretopology.mem_sInf (C : Type u) [Category.{v, u} C] [Limits.HasPullbacks C] (T : Set (Pretopology C)) {X : C} (S : Presieve X) :
              S (sInf T).coverings X tT, S t.coverings X

              The complete lattice structure on pretopologies. This is induced by the InfSet instance, but with good definitional equalities for , and .

              Equations
              • One or more equations did not get rendered due to their size.
              theorem CategoryTheory.Pretopology.mem_inf (C : Type u) [Category.{v, u} C] [Limits.HasPullbacks C] (t₁ t₂ : Pretopology C) {X : C} (S : Presieve X) :
              S (t₁t₂).coverings X S t₁.coverings X S t₂.coverings X

              If J is a precoverage that has isomorphisms and is stable under composition and base change, it defines a pretopology.

              Equations
              Instances For