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'
.
noncomputable def
PresheafOfModules.restrictScalarsObj
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(M' : PresheafOfModules R')
(α : R ⟶ R')
:
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.restrictScalarsObj_map
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(M' : PresheafOfModules R')
(α : R ⟶ R')
{X Y : Cᵒᵖ}
(f : X ⟶ Y)
:
(M'.restrictScalarsObj α).map f = ModuleCat.ofHom { toFun := ⇑(CategoryTheory.ConcreteCategory.hom (M'.map f)), map_add' := ⋯, map_smul' := ⋯ }
@[simp]
theorem
PresheafOfModules.restrictScalarsObj_obj
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(M' : PresheafOfModules R')
(α : R ⟶ R')
(X : Cᵒᵖ)
:
(M'.restrictScalarsObj α).obj X = (ModuleCat.restrictScalars (RingCat.Hom.hom (α.app X))).obj (M'.obj X)
noncomputable def
PresheafOfModules.restrictScalars
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(α : R ⟶ R')
:
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
@[simp]
theorem
PresheafOfModules.restrictScalars_obj
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(α : R ⟶ R')
(M' : PresheafOfModules R')
:
@[simp]
theorem
PresheafOfModules.restrictScalars_map_app
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(α : R ⟶ R')
{X✝ Y✝ : PresheafOfModules R'}
(φ' : X✝ ⟶ Y✝)
(X : Cᵒᵖ)
:
((restrictScalars α).map φ').app X = (ModuleCat.restrictScalars (RingCat.Hom.hom (α.app X))).map (φ'.app X)
instance
PresheafOfModules.instAdditiveRestrictScalars
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(α : R ⟶ R')
:
instance
PresheafOfModules.instFaithfulRestrictScalars
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(α : R ⟶ R')
:
noncomputable def
PresheafOfModules.restrictScalarsCompToPresheaf
{C : Type u'}
[CategoryTheory.Category.{v', u'} C]
{R R' : CategoryTheory.Functor Cᵒᵖ RingCat}
(α : R ⟶ R')
:
The isomorphism restrictScalars α ⋙ toPresheaf R ≅ toPresheaf R'
for any
morphism of presheaves of rings α : R ⟶ R'
.