Ideals in localizations of commutative rings #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Implementation notes #
See src/ring_theory/localization/basic.lean
for a design overview.
Tags #
localization, ring localization, commutative ring localization, characteristic predicate, commutative ring, field of fractions
If S
is the localization of R
at a submonoid, the ordering of ideals of S
is
embedded in the ordering of ideals of R
.
Equations
- is_localization.order_embedding M S = {to_embedding := {to_fun := λ (J : ideal S), ideal.comap (algebra_map R S) J, inj' := _}, map_rel_iff' := _}
If R
is a ring, then prime ideals in the localization at M
correspond to prime ideals in the original ring R
that are disjoint from M
.
This lemma gives the particular case for an ideal and its comap,
see le_rel_iso_of_prime
for the more general relation isomorphism
If R
is a ring, then prime ideals in the localization at M
correspond to prime ideals in the original ring R
that are disjoint from M
.
This lemma gives the particular case for an ideal and its map,
see le_rel_iso_of_prime
for the more general relation isomorphism, and the reverse implication
If R
is a ring, then prime ideals in the localization at M
correspond to prime ideals in the original ring R
that are disjoint from M
Equations
- is_localization.order_iso_of_prime M S = {to_equiv := {to_fun := λ (p : {p // p.is_prime}), ⟨ideal.comap (algebra_map R S) p.val, _⟩, inv_fun := λ (p : {p // p.is_prime ∧ disjoint ↑M ↑p}), ⟨ideal.map (algebra_map R S) p.val, _⟩, left_inv := _, right_inv := _}, map_rel_iff' := _}
quotient_map
applied to maximal ideals of a localization is surjective
.
The quotient by a maximal ideal is a field, so inverses to elements already exist,
and the localization necessarily maps the equivalence class of the inverse in the localization