Documentation

Mathlib.CategoryTheory.Sites.InducedTopology

Induced Topology #

We say that a functor G : C ⥤ (D, K) is locally dense if for each covering sieve T in D of some X : C, T ∩ mor(C) generates a covering sieve of X in D. A locally dense fully faithful functor then induces a topology on C via { T ∩ mor(C) | T ∈ K }. Note that this is equal to the collection of sieves on C whose image generates a covering sieve. This construction would make C both cover-lifting and cover-preserving.

Some typical examples are full and cover-dense functors (for example the functor from a basis of a topological space X into Opens X). The functor Over X ⥤ C is also locally dense, and the induced topology can then be used to construct the big sites associated to a scheme.

Given a fully faithful cover-dense functor G : C ⥤ (D, K) between small sites, we then have Sheaf (H.inducedTopology) A ≌ Sheaf K A. This is known as the comparison lemma.

References #

We say that a functor C ⥤ D into a site is "locally dense" if for each covering sieve T in D, T ∩ mor(C) generates a covering sieve in D.

Equations
Instances For

    If a functor G : C ⥤ (D, K) is fully faithful and locally dense, then the set { T ∩ mor(C) | T ∈ K } is a grothendieck topology of C.

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

      G is cover-lifting wrt the induced topology.

      @[reducible, inline]

      Given a fully faithful cover-dense functor G : C ⥤ (D, K), we may induce a topology on C.

      Equations
      • G.inducedTopologyOfIsCoverDense K = .inducedTopology
      Instances For
        instance CategoryTheory.instIsContinuousInducedTopologyOfIsCoverDense {C : Type v} [CategoryTheory.SmallCategory C] {D : Type v} [CategoryTheory.SmallCategory D] {G : CategoryTheory.Functor C D} {K : CategoryTheory.GrothendieckTopology D} [G.Full] [G.Faithful] [G.IsCoverDense K] :
        G.IsContinuous (G.inducedTopologyOfIsCoverDense K) K
        Equations
        • =
        instance CategoryTheory.instIsCocontinuousInducedTopologyOfIsCoverDense {C : Type v} [CategoryTheory.SmallCategory C] {D : Type v} [CategoryTheory.SmallCategory D] {G : CategoryTheory.Functor C D} {K : CategoryTheory.GrothendieckTopology D} [G.Full] [G.Faithful] [G.IsCoverDense K] :
        G.IsCocontinuous (G.inducedTopologyOfIsCoverDense K) K
        Equations
        • =

        Cover-dense functors induces an equivalence of categories of sheaves.

        This is known as the comparison lemma. It requires that the sites are small and the value category is complete.

        Equations
        Instances For