Documentation

Mathlib.CategoryTheory.Sites.Pullback

Pullback of sheaves #

Main definitions #

The pullback functor Sheaf J A ⥤ Sheaf K A associated to a functor G : C ⥤ D in the same direction as G.

Equations
  • G.sheafPullback A J K = (G.sheafPushforwardContinuous A J K).leftAdjoint
Instances For
    def CategoryTheory.Functor.sheafAdjunctionContinuous {C : Type u₂} [CategoryTheory.Category.{v₂, u₂} C] {D : Type u₃} [CategoryTheory.Category.{v₃, u₃} D] (G : CategoryTheory.Functor C D) (A : Type u₁) [CategoryTheory.Category.{v₁, u₁} A] (J : CategoryTheory.GrothendieckTopology C) (K : CategoryTheory.GrothendieckTopology D) [G.IsContinuous J K] [(G.sheafPushforwardContinuous A J K).IsRightAdjoint] :
    G.sheafPullback A J K G.sheafPushforwardContinuous A J K

    The pullback functor is left adjoint to the pushforward functor.

    Equations
    Instances For

      The constructed sheafPullback G A J K is left adjoint to G.sheafPushforwardContinuous A J K.

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

        The constructed pullback of sheaves is isomorphic to the abstract one.

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