Henselian rings #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we set up the basic theory of Henselian (local) rings.
A ring R is Henselian at an ideal I if the following conditions hold:
Iis contained in the Jacobson radical ofR- for every polynomial
foverR, with a simple roota₀over the quotient ringR/I, there exists a lifta : Rofa₀that is a root off.
(Here, saying that a root b of a polynomial g is simple means that g.derivative.eval b is a
unit. Warning: if R/I is not a field then it is not enough to assume that g has a factorization
into monic linear factors in which X - b shows up only once; for example 1 is not a simple root
of X^2-1 over ℤ/4ℤ.)
A local ring R is Henselian if it is Henselian at its maximal ideal.
In this case the first condition is automatic, and in the second condition we may ask for
f.derivative.eval a ≠ 0, since the quotient ring R/I is a field in this case.
Main declarations #
henselian_ring: a typeclass on commutative rings, asserting that the ring is Henselian at the idealI.henselian_local_ring: a typeclass on commutative rings, asserting that the ring is local Henselian.field.henselian: fields are Henselian local ringshenselian.tfae: equivalent ways of expressing the Henselian property for local ringsis_adic_complete.henselian: a ringRwith idealIthat isI-adically complete is Henselian atI
References #
https://stacks.math.columbia.edu/tag/04GE
Todo #
After a good API for etale ring homomorphisms has been developed, we can give more equivalent characterization os Henselian rings.
In particular, this can give a proof that factorizations into coprime polynomials can be lifted from the residue field to the Henselian ring.
The following gist contains some code sketches in that direction. https://gist.github.com/jcommelin/47d94e4af092641017a97f7f02bf9598
- jac : I ≤ ⊥.jacobson
- is_henselian : ∀ (f : polynomial R), f.monic → ∀ (a₀ : R), polynomial.eval a₀ f ∈ I → is_unit (⇑(ideal.quotient.mk I) (polynomial.eval a₀ (⇑polynomial.derivative f))) → (∃ (a : R), f.is_root a ∧ a - a₀ ∈ I)
A ring R is Henselian at an ideal I if the following condition holds:
for every polynomial f over R, with a simple root a₀ over the quotient ring R/I,
there exists a lift a : R of a₀ that is a root of f.
(Here, saying that a root b of a polynomial g is simple means that g.derivative.eval b is a
unit. Warning: if R/I is not a field then it is not enough to assume that g has a factorization
into monic linear factors in which X - b shows up only once; for example 1 is not a simple root
of X^2-1 over ℤ/4ℤ.)
Instances of this typeclass
- to_local_ring : local_ring R
- is_henselian : ∀ (f : polynomial R), f.monic → ∀ (a₀ : R), polynomial.eval a₀ f ∈ local_ring.maximal_ideal R → is_unit (polynomial.eval a₀ (⇑polynomial.derivative f)) → (∃ (a : R), f.is_root a ∧ a - a₀ ∈ local_ring.maximal_ideal R)
A local ring R is Henselian if the following condition holds:
for every polynomial f over R, with a simple root a₀ over the residue field,
there exists a lift a : R of a₀ that is a root of f.
(Recall that a root b of a polynomial g is simple if it is not a double root, so if
g.derivative.eval b ≠ 0.)
In other words, R is local Henselian if it is Henselian at the ideal I,
in the sense of henselian_ring.
Instances of this typeclass
A ring R that is I-adically complete is Henselian at I.