Integral and algebraic elements of a fraction field #
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
coeff_integer_normalization p
gives the coefficients of the polynomial
integer_normalization p
Equations
- is_localization.coeff_integer_normalization M p i = dite (i ∈ p.support) (λ (hi : i ∈ p.support), classical.some _) (λ (hi : i ∉ p.support), 0)
integer_normalization g
normalizes g
to have integer coefficients
by clearing the denominators
Equations
- is_localization.integer_normalization M p = p.support.sum (λ (i : ℕ), ⇑(polynomial.monomial i) (is_localization.coeff_integer_normalization M p i))
An element of a ring is algebraic over the ring A
iff it is algebraic
over the field of fractions of A
.
A ring is algebraic over the ring A
iff it is algebraic over the field of fractions of A
.
Given a particular witness to an element being algebraic over an algebra R → S
,
We can localize to a submonoid containing the leading coefficient to make it integral.
Explicitly, the map between the localizations will be an integral ring morphism
If R → S
is an integral extension, M
is a submonoid of R
,
Rₘ
is the localization of R
at M
,
and Sₘ
is the localization of S
at the image of M
under the extension map,
then the induced map Rₘ → Sₘ
is also an integral extension
If the field L
is an algebraic extension of the integral domain A
,
the integral closure C
of A
in L
has fraction field L
.
If the field L
is a finite extension of the fraction field of the integral domain A
,
the integral closure C
of A
in L
has fraction field L
.
If the field L
is an algebraic extension of the integral domain A
,
the integral closure of A
in L
has fraction field L
.
If the field L
is a finite extension of the fraction field of the integral domain A
,
the integral closure of A
in L
has fraction field L
.
S
is algebraic over R
iff a fraction ring of S
is algebraic over R
If the S
-multiples of a
are contained in some R
-span, then Frac(S)
-multiples of a
are contained in the equivalent Frac(R)
-span.