Integral closure of a subring.
If A is an R-algebra then a : A is integral over R if it is a root of a monic polynomial
with coefficients in R. Enough theory is developed to prove that integral elements
form a sub-R-algebra of A.
Main definitions
Let R be a comm_ring and let A be an R-algebra.
ring_hom.is_integral_elem (f : R →+* A) (x : A):xis integral with respect to the mapf,is_integral (x : A):xis integral overR, i.e., is a root of a monic polynomial with coefficients inR.integral_closure R A: the integral closure ofRinA, regarded as a sub-R-algebra ofA.
An element x of A is said to be integral over R with respect to f
if it is a root of a monic polynomial p : polynomial R evaluated under f
Equations
- f.is_integral_elem x = ∃ (p : polynomial R), p.monic ∧ polynomial.eval₂ f x p = 0
A ring homomorphism f : R →+* A is said to be integral
if every element A is integral with respect to the map f
Equations
- f.is_integral = ∀ (x : A), f.is_integral_elem x
An element x of an algebra A over a commutative ring R is said to be integral,
if it is a root of some monic polynomial p : polynomial R.
Equivalently, the element is integral over R with respect to the induced algebra_map
Equations
- is_integral R x = (algebra_map R A).is_integral_elem x
An algebra is integral if every element of the extension is integral over the base ring
Equations
- algebra.is_integral R A = (algebra_map R A).is_integral
The integral closure of R in an R-algebra A.
Equations
- integral_closure R A = {carrier := {r : A | is_integral R r}, one_mem' := _, mul_mem' := _, zero_mem' := _, add_mem' := _, algebra_map_mem' := _}
Mapping an integral closure along an alg_equiv gives the integral closure.
If A is an R-algebra all of whose elements are integral over R, and x is an element of an A-algebra that is integral over A, then x is integral over R.
If A is an R-algebra all of whose elements are integral over R, and B is an A-algebra all of whose elements are integral over A, then all elements of B are integral over R.
If R → A → B is an algebra tower with A → B injective,
then if the entire tower is an integral extension so is R → A
If R → A → B is an algebra tower,
then if the entire tower is an integral extension so is A → B
If the integral extension R → S is injective, and S is a field, then R is also a field
Equations
- integral_closure.integral_domain = {add := comm_ring.add (subalgebra.comm_ring R S (integral_closure R S)), add_assoc := _, zero := comm_ring.zero (subalgebra.comm_ring R S (integral_closure R S)), zero_add := _, add_zero := _, neg := comm_ring.neg (subalgebra.comm_ring R S (integral_closure R S)), add_left_neg := _, add_comm := _, mul := comm_ring.mul (subalgebra.comm_ring R S (integral_closure R S)), mul_assoc := _, one := comm_ring.one (subalgebra.comm_ring R S (integral_closure R S)), one_mul := _, mul_one := _, left_distrib := _, right_distrib := _, mul_comm := _, exists_pair_ne := _, eq_zero_or_eq_zero_of_mul_eq_zero := _}