Change Of Rings #
Main definitions #
-
ModuleCat.restrictScalars: given ringsR, Sand a ring homomorphismR ⟶ S, thenrestrictScalars : ModuleCat S ⥤ ModuleCat Ris defined byM ↦ Mwhere anS-moduleMis seen as anR-module byr • m := f r • mandS-linear mapl : M ⟶ M'isR-linear as well. -
ModuleCat.extendScalars: given commutative ringsR, Sand ring homomorphismf : R ⟶ S, thenextendScalars : ModuleCat R ⥤ ModuleCat Sis defined byM ↦ S ⨂ Mwhere the module structure is defined bys • (s' ⊗ m) := (s * s') ⊗ mandR-linear mapl : M ⟶ M'is sent toS-linear maps ⊗ m ↦ s ⊗ l m : S ⨂ M ⟶ S ⨂ M'. -
ModuleCat.coextendScalars: given ringsR, Sand a ring homomorphismR ⟶ SthencoextendScalars : ModuleCat R ⥤ ModuleCat Sis defined byM ↦ (S →ₗ[R] M)whereSis seen as anR-module by restriction of scalars andl ↦ l ∘ _.
Main results #
ModuleCat.extendRestrictScalarsAdj: given commutative ringsR, Sand a ring homomorphismf : R →+* S, the extension and restriction of scalars byfare adjoint functors.ModuleCat.restrictCoextendScalarsAdj: given ringsR, Sand a ring homomorphismf : R ⟶ SthencoextendScalars fis the right adjoint ofrestrictScalars f.
List of notations #
Let R, S be rings and f : R →+* S
- if
Mis anR-module,s : Sandm : M, thens ⊗ₜ[R, f] mis the pure tensors ⊗ m : S ⊗[R, f] M.
Any S-module M is also an R-module via a ring homomorphism f : R ⟶ S by defining
r • m := f r • m (Module.compHom). This is called restriction of scalars.
Equations
Instances For
Given an S-linear map g : M → M' between S-modules, g is also R-linear between M and
M' by means of restriction of scalars.
Equations
- ModuleCat.RestrictScalars.map' f g = { toAddHom := g.toAddHom, map_smul' := (_ : ∀ (r : R) (x : ↑M), g (f r • x) = f r • g x) }
Instances For
The restriction of scalars operation is functorial. For any f : R →+* S a ring homomorphism,
- an
S-moduleMcan be considered asR-module byr • m = f r • m - an
S-linear map is alsoR-linear
Equations
- ModuleCat.restrictScalars f = CategoryTheory.Functor.mk { obj := ModuleCat.RestrictScalars.obj' f, map := fun {X Y : ModuleCat S} => ModuleCat.RestrictScalars.map' f }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- (_ : SMulCommClass R S M) = (_ : SMulCommClass R S M)
Semilinear maps M →ₛₗ[f] N identify to
morphisms M ⟶ (ModuleCat.restrictScalars f).obj N.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The restriction of scalars by a ring morphism that is the identity identify to the identity functor.
Equations
- ModuleCat.restrictScalarsId' f hf = (_ : RingHom.id R = f) ▸ CategoryTheory.Iso.refl (ModuleCat.restrictScalars (RingHom.id R))
Instances For
The restriction of scalars by the identity morphisms identify to the identity functor.
Equations
- ModuleCat.restrictScalarsId R = ModuleCat.restrictScalarsId' (RingHom.id R) (_ : RingHom.id R = RingHom.id R)
Instances For
The restriction of scalars by a composition of ring morphisms identify to the composition of the restriction of scalars functors.
Equations
- ModuleCat.restrictScalarsComp' f g gf hgf = (_ : RingHom.comp g f = gf) ▸ CategoryTheory.Iso.refl (ModuleCat.restrictScalars (RingHom.comp g f))
Instances For
The restriction of scalars by a composition of ring morphisms identify to the composition of the restriction of scalars functors.
Equations
- ModuleCat.restrictScalarsComp f g = ModuleCat.restrictScalarsComp' f g (RingHom.comp g f) (_ : RingHom.comp g f = RingHom.comp g f)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Extension of scalars turn an R-module into S-module by M ↦ S ⨂ M
Equations
- ModuleCat.ExtendScalars.obj' f M = ModuleCat.mk (TensorProduct R ↑((ModuleCat.restrictScalars f).toPrefunctor.obj (ModuleCat.mk S)) ↑M)
Instances For
Extension of scalars is a functor where an R-module M is sent to S ⊗ M and
l : M1 ⟶ M2 is sent to s ⊗ m ↦ s ⊗ l m
Equations
Instances For
Extension of scalars is a functor where an R-module M is sent to S ⊗ M and
l : M1 ⟶ M2 is sent to s ⊗ m ↦ s ⊗ l m
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given an R-module M, consider Hom(S, M) -- the R-linear maps between S (as an R-module by
means of restriction of scalars) and M. S acts on Hom(S, M) by s • g = x ↦ g (x • s)
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
S acts on Hom(S, M) by s • g = x ↦ g (x • s), this action defines an S-module structure on
Hom(S, M).
Equations
- One or more equations did not get rendered due to their size.
If M is an R-module, then the set of R-linear maps S →ₗ[R] M is an S-module with
scalar multiplication defined by s • l := x ↦ l (x • s)
Equations
- ModuleCat.CoextendScalars.obj' f M = ModuleCat.mk (↑((ModuleCat.restrictScalars f).toPrefunctor.obj (ModuleCat.mk S)) →ₗ[R] ↑M)
Instances For
Equations
- ModuleCat.CoextendScalars.instCoeFunCarrierObj'ForAllCarrier f M = { coe := fun (g : ↑(ModuleCat.CoextendScalars.obj' f M)) => g.toFun }
If M, M' are R-modules, then any R-linear map g : M ⟶ M' induces an S-linear map
(S →ₗ[R] M) ⟶ (S →ₗ[R] M') defined by h ↦ g ∘ h
Equations
- One or more equations did not get rendered due to their size.
Instances For
For any rings R, S and a ring homomorphism f : R →+* S, there is a functor from R-module to
S-module defined by M ↦ (S →ₗ[R] M) where S is considered as an R-module via restriction of
scalars and g : M ⟶ M' is sent to h ↦ g ∘ h.
Equations
- ModuleCat.coextendScalars f = CategoryTheory.Functor.mk { obj := ModuleCat.CoextendScalars.obj' f, map := fun {X Y : ModuleCat R} => ModuleCat.CoextendScalars.map' f }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Given R-module X and S-module Y, any g : (restrictScalars f).obj Y ⟶ X
corresponds to Y ⟶ (coextendScalars f).obj X by sending y ↦ (s ↦ g (s • y))
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given R-module X and S-module Y, any g : Y ⟶ (coextendScalars f).obj X
corresponds to (restrictScalars f).obj Y ⟶ X by y ↦ g y 1
Equations
- One or more equations did not get rendered due to their size.
Instances For
Auxiliary definition for unit'
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural transformation from the composition of coextension and restriction of scalars to identity functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given R-module X and S-module Y and a map g : (extendScalars f).obj X ⟶ Y, i.e. S-linear
map S ⨂ X → Y, there is a X ⟶ (restrictScalars f).obj Y, i.e. R-linear map X ⟶ Y by
x ↦ g (1 ⊗ x).
Equations
- One or more equations did not get rendered due to their size.
Instances For
The map S → X →ₗ[R] Y given by fun s x => s • (g x)
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given R-module X and S-module Y and a map X ⟶ (restrictScalars f).obj Y, i.e R-linear map
X ⟶ Y, there is a map (extend_scalars f).obj X ⟶ Y, i.e S-linear map S ⨂ X → Y by
s ⊗ x ↦ s • g x.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given R-module X and S-module Y, S-linear linear maps (extendScalars f).obj X ⟶ Y
bijectively correspond to R-linear maps X ⟶ (restrictScalars f).obj Y.
Equations
- One or more equations did not get rendered due to their size.
Instances For
For any R-module X, there is a natural R-linear map from X to X ⨂ S by sending x ↦ x ⊗ 1
Equations
- One or more equations did not get rendered due to their size.
Instances For
For any S-module Y, there is a natural R-linear map from S ⨂ Y to Y by
s ⊗ y ↦ s • y
Instances For
Given commutative rings R, S and a ring hom f : R →+* S, the extension and restriction of
scalars by f are adjoint to each other.
Equations
- One or more equations did not get rendered due to their size.