Documentation

Mathlib.CategoryTheory.Sites.CoverPreserving

Cover-preserving and continuous functors between sites. #

We define the notion of continuous functor between sites: these are functors G such that the precomposition with G.op preserves sheaves of types (and actually sheaves in any category).

In order to show that a functor is continuous, we define cover-preserving functors between sites as functors that push covering sieves to covering sieves. Then, a cover-preserving and compatible-preserving functor is continuous.

Main definitions #

Main results #

References #

A functor G : (C, J) ⥤ (D, K) between sites is cover-preserving if for all covering sieves R in C, R.functorPushforward G is a covering sieve in D.

Instances For

    A functor G : (C, J) ⥤ (D, K) between sites is called compatible preserving if for each compatible family of elements at C and valued in G.op ⋙ ℱ, and each commuting diagram f₁ ≫ G.map g₁ = f₂ ≫ G.map g₂, x g₁ and x g₂ coincide when restricted via fᵢ. This is actually stronger than merely preserving compatible families because of the definition of functorPushforward used.

    Instances For

      A functor F is continuous if the precomposition with F.op sends sheaves of Type w to sheaves.

      Instances

        The induced functor Sheaf K A ⥤ Sheaf J A given by G.op ⋙ _ if G is a continuous functor.

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