Documentation

Mathlib.Algebra.Category.ModuleCat.Presheaf.Sheafify

The associated sheaf of a presheaf of modules #

In this file, given a presheaf of modules M₀ over a presheaf of rings R₀, we construct the associated sheaf of M₀. More precisely, if R is a sheaf of rings and α : R₀ ⟶ R.val is locally bijective, and A is the sheafification of the underlying presheaf of abelian groups of M₀, i.e. we have a locally bijective map φ : M₀.presheaf ⟶ A.val, then we endow A with the structure of a sheaf of modules over R: this is PresheafOfModules.sheafify α φ.

In many applications, the morphism α shall be the identity, but this more general construction allows the sheafification of both the presheaf of rings and the presheaf of modules.

The scalar multiplication of family of elements of a presheaf of modules M over R by a family of elements of R.

Equations
Instances For
    theorem CategoryTheory.Presieve.FamilyOfElements.isCompatible_map_smul_aux {C : Type u₁} [Category.{v₁, u₁} C] {J : GrothendieckTopology C} {R₀ R : Functor Cᵒᵖ RingCat} (α : R₀ R) [Presheaf.IsLocallyInjective J α] {M₀ : PresheafOfModules R₀} {A : Functor Cᵒᵖ AddCommGrp} (φ : M₀.presheaf A) [Presheaf.IsLocallyInjective J φ] (hA : Presheaf.IsSeparated J A) {X : C} (r : (R.obj (Opposite.op X))) (m : (A.obj (Opposite.op X))) {Y Z : C} (f : Y X) (g : Z Y) (r₀ : (R₀.obj (Opposite.op Y))) (r₀' : (R₀.obj (Opposite.op Z))) (m₀ : (M₀.obj (Opposite.op Y))) (m₀' : (M₀.obj (Opposite.op Z))) (hr₀ : (ConcreteCategory.hom (α.app (Opposite.op Y))) r₀ = (ConcreteCategory.hom (R.map f.op)) r) (hr₀' : (ConcreteCategory.hom (α.app (Opposite.op Z))) r₀' = (ConcreteCategory.hom (R.map (CategoryStruct.comp f.op g.op))) r) (hm₀ : (ConcreteCategory.hom (φ.app (Opposite.op Y))) m₀ = (ConcreteCategory.hom (A.map f.op)) m) (hm₀' : (ConcreteCategory.hom (φ.app (Opposite.op Z))) m₀' = (ConcreteCategory.hom (A.map (CategoryStruct.comp f.op g.op))) m) :
    (ConcreteCategory.hom (φ.app (Opposite.op Z))) ((ConcreteCategory.hom (M₀.map g.op)) (r₀ m₀)) = (ConcreteCategory.hom (φ.app (Opposite.op Z))) (r₀' m₀')
    theorem CategoryTheory.Presieve.FamilyOfElements.isCompatible_map_smul {C : Type u₁} [Category.{v₁, u₁} C] {J : GrothendieckTopology C} {R₀ R : Functor Cᵒᵖ RingCat} (α : R₀ R) [Presheaf.IsLocallyInjective J α] {M₀ : PresheafOfModules R₀} {A : Functor Cᵒᵖ AddCommGrp} (φ : M₀.presheaf A) [Presheaf.IsLocallyInjective J φ] (hA : Presheaf.IsSeparated J A) {X : C} (r : (R.obj (Opposite.op X))) (m : (A.obj (Opposite.op X))) {P : Presieve X} (r₀ : FamilyOfElements (R₀.comp (forget RingCat)) P) (m₀ : FamilyOfElements (M₀.presheaf.comp (forget Ab)) P) (hr₀ : (r₀.map (whiskerRight α (forget RingCat))).IsAmalgamation r) (hm₀ : (m₀.map (whiskerRight φ (forget Ab))).IsAmalgamation m) :
    ((r₀.smul m₀).map (whiskerRight φ (forget Ab))).Compatible

    Assuming α : R₀ ⟶ R.val is the sheafification map of a presheaf of rings R₀ and φ : M₀.presheaf ⟶ A.val is the sheafification map of the underlying sheaf of abelian groups of a presheaf of modules M₀ over R₀, then given r : R.val.obj X and m : A.val.obj X, this structure contains the data of x : A.val.obj X along with the property which makes x a good candidate for the definition of the scalar multiplication r • m.

    Instances For

      The module structure on the sections of the sheafification of the underlying presheaf of abelian groups of a presheaf of modules.

      Equations
      Instances For

        Assuming α : R₀ ⟶ R.val is the sheafification map of a presheaf of rings R₀ and φ : M₀.presheaf ⟶ A.val is the sheafification map of the underlying sheaf of abelian groups of a presheaf of modules M₀ over R₀, this is the sheaf of modules over R which is obtained by endowing the sections of A.val with a scalar multiplication.

        Equations
        Instances For

          The bijection ((sheafify α φ).val ⟶ F) ≃ (M₀ ⟶ (restrictScalars α).obj F) which is part of the universal property of the sheafification of the presheaf of modules M₀, when F is a presheaf of modules which is a sheaf.

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

            The bijection (sheafify α φ ⟶ F) ≃ (M₀ ⟶ (restrictScalars α).obj ((SheafOfModules.forget _).obj F)) which is part of the universal property of the sheafification of the presheaf of modules M₀, for any sheaf of modules F, see PresheafOfModules.sheafificationAdjunction

            Equations
            Instances For

              The morphism of sheaves of modules sheafify α φ ⟶ sheafify α φ' induced by morphisms τ₀ : M₀ ⟶ M₀' and τ : A ⟶ A' which satisfy τ₀.hom ≫ φ' = φ ≫ τ.val.

              Equations
              Instances For