Localizations of commutative rings at the complement of a prime ideal #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Main definitions #
is_localization.at_prime (I : ideal R) [is_prime I] (S : Type*)
expresses thatS
is a localization at (the complement of) a prime idealI
, as an abbreviation ofis_localization I.prime_compl S
Main results #
is_localization.at_prime.local_ring
: a theorem (not an instance) stating a localization at the complement of a prime ideal is a local ring
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
The complement of a prime ideal I ⊆ R
is a submonoid of R
.
Instances for ideal.prime_compl
- is_localization.localization_localization_at_prime_is_localization
- valuation_subring.of_prime_localization
- algebraic_geometry.structure_sheaf.as_ideal.is_localization.at_prime
- algebraic_geometry.structure_sheaf.is_localization.to_stalk
- algebraic_geometry.structure_sheaf.is_localized_module_to_pushforward_stalk_alg_hom
Given a prime ideal P
, the typeclass is_localization.at_prime S P
states that S
is
isomorphic to the localization of R
at the complement of P
.
Given a prime ideal P
, localization.at_prime S P
is a localization of
R
at the complement of P
, as a quotient type.
The localization of R
at the complement of a prime ideal is a local ring.
The unique maximal ideal of the localization at I.prime_compl
lies over the ideal I
.
The image of I
in the localization at I.prime_compl
is a maximal ideal, and in particular
it is the unique maximal ideal given by the local ring structure at_prime.local_ring
For a ring hom f : R →+* S
and a prime ideal J
in S
, the induced ring hom from the
localization of R
at J.comap f
to the localization of S
at J
.
To make this definition more flexible, we allow any ideal I
of R
as input, together with a proof
that I = J.comap f
. This can be useful when I
is not definitionally equal to J.comap f
.
Equations
- localization.local_ring_hom I J f hIJ = is_localization.map (localization.at_prime J) f _