Documentation

Mathlib.Algebra.Category.ModuleCat.Sheaf

Sheaves of modules over a sheaf of rings #

In this file, we define the category SheafOfModules R when R : Sheaf J RingCat is a sheaf of rings on a category C equipped with a Grothendieck topology J.

TODO #

structure SheafOfModules {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {J : CategoryTheory.GrothendieckTopology C} (R : CategoryTheory.Sheaf J RingCat) :
Type (max (max (max u u₁) (v + 1)) v₁)

A sheaf of modules is a presheaf of modules such that the underlying presheaf of abelian groups is a sheaf.

Instances For
    theorem SheafOfModules.Hom.ext {C : Type u₁} :
    ∀ {inst : CategoryTheory.Category.{v₁, u₁} C} {J : CategoryTheory.GrothendieckTopology C} {R : CategoryTheory.Sheaf J RingCat} {X Y : SheafOfModules R} (x y : X.Hom Y), x.val = y.valx = y
    theorem SheafOfModules.Hom.ext_iff {C : Type u₁} :
    ∀ {inst : CategoryTheory.Category.{v₁, u₁} C} {J : CategoryTheory.GrothendieckTopology C} {R : CategoryTheory.Sheaf J RingCat} {X Y : SheafOfModules R} (x y : X.Hom Y), x = y x.val = y.val

    A morphism between sheaves of modules is a morphism between the underlying presheaves of modules.

    • val : X.val Y.val

      a morphism between the underlying presheaves of modules

    Instances For

      The forgetful functor SheafOfModules.{v} R ⥤ PresheafOfModules R.val.

      Equations
      Instances For