Documentation

Mathlib.Algebra.Category.ModuleCat.Presheaf.Sheafification

The sheafification functor for presheaves of modules #

In this file, we construct a functor PresheafOfModules.sheafification α : PresheafOfModules R₀ ⥤ SheafOfModules R for a locally bijective morphism α : R₀ ⟶ R.val where R₀ is a presheaf of rings and R a sheaf of rings. In particular, if α is the identity of R.val, we obtain the sheafification functor PresheafOfModules R.val ⥤ SheafOfModules R.

Given a locally bijective morphism α : R₀ ⟶ R.val where R₀ is a presheaf of rings and R a sheaf of rings (i.e. R identifies to the sheafification of R₀), this is the associated sheaf of modules functor PresheafOfModules.{v} R₀ ⥤ SheafOfModules.{v} R.

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

    The sheafification of presheaves of modules commutes with the functor which forgets the module structures.

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

      Given a locally bijective morphism α : R₀ ⟶ R.val where R₀ is a presheaf of rings and R a sheaf of rings, this is the adjunction sheafification.{v} α ⊣ SheafOfModules.forget R ⋙ restrictScalars α.

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