Documentation

Mathlib.Algebra.Category.ModuleCat.Presheaf.ChangeOfRings

Change of presheaf of rings #

In this file, we define the restriction of scalars functor restrictScalars α : PresheafOfModules.{v} R' ⥤ PresheafOfModules.{v} R attached to a morphism of presheaves of rings α : R ⟶ R'.

@[simp]
theorem PresheafOfModules.restrictScalarsBundledCore_map_apply {C : Type u'} [CategoryTheory.Category.{v', u'} C] {R : CategoryTheory.Functor Cᵒᵖ RingCat} {R' : CategoryTheory.Functor Cᵒᵖ RingCat} (M' : PresheafOfModules R') (α : R R') {X : Cᵒᵖ} {Y : Cᵒᵖ} (f : X Y) (a : (M'.obj X)) :
((M'.restrictScalarsBundledCore α).map f) a = (M'.map f) a
@[simp]
theorem PresheafOfModules.restrictScalarsBundledCore_obj {C : Type u'} [CategoryTheory.Category.{v', u'} C] {R : CategoryTheory.Functor Cᵒᵖ RingCat} {R' : CategoryTheory.Functor Cᵒᵖ RingCat} (M' : PresheafOfModules R') (α : R R') (X : Cᵒᵖ) :
(M'.restrictScalarsBundledCore α).obj X = (ModuleCat.restrictScalars (α.app X)).obj (M'.obj X)

The restriction of scalars of presheaves of modules, on objects.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem PresheafOfModules.restrictScalars_obj {C : Type u'} [CategoryTheory.Category.{v', u'} C] {R : CategoryTheory.Functor Cᵒᵖ RingCat} {R' : CategoryTheory.Functor Cᵒᵖ RingCat} (α : R R') (M' : PresheafOfModules R') :
    (PresheafOfModules.restrictScalars α).obj M' = (M'.restrictScalarsBundledCore α).toPresheafOfModules

    The restriction of scalars functor PresheafOfModules R' ⥤ PresheafOfModules R induced by a morphism of presheaves of rings R ⟶ R'.

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