Localized Module #
Given a commutative semiring R
, a multiplicative subset S ⊆ R
and an R
-module M
, we can
localize M
by S
. This gives us a Localization S
-module.
Main definition #
isLocalizedModule_iff_isBaseChange
: A localization of modules corresponds to a base change.
The forward direction of isLocalizedModule_iff_isBaseChange
. It is also used to prove the
other direction.
The map (f : M →ₗ[R] M')
is a localization of modules iff the map
(Localization S) × M → N, (s, m) ↦ s • f m
is the tensor product (insomuch as it is the universal
bilinear map).
In particular, there is an isomorphism between LocalizedModule S M
and (Localization S) ⊗[R] M
given by m/s ↦ (1/s) ⊗ₜ m
.
If A
is a localization of R
, tensoring two A
-modules over A
is the same as
tensoring them over R
.
Equations
- IsLocalization.moduleTensorEquiv S A M₁ M₂ = TensorProduct.equivOfCompatibleSMul R A M₁ M₂
Instances For
If A
is a localization of R
, tensoring an A
-module with A
over R
does nothing.
Equations
- IsLocalization.moduleLid S A M₁ = (TensorProduct.equivOfCompatibleSMul R A A M₁).symm.trans (TensorProduct.lid A M₁)
Instances For
If A
is a localization of R
, tensoring two A
-algebras over A
is the same as
tensoring them over R
.
Equations
Instances For
If A
is a localization of R
, tensoring an A
-algebra with A
over R
does nothing.
Equations
Instances For
Alias of IsLocalization.algebraLid
.
If A
is a localization of R
, tensoring an A
-algebra with A
over R
does nothing.
Instances For
S⁻¹M ⊗[R] N = S⁻¹(M ⊗[R] N)
.