The spectral norm and the norm extension theorem #
This file shows that if K is a nonarchimedean normed field and L/K is an algebraic extension,
then there is a natural extension of the norm on K to a K-algebra norm on L, the so-called
spectral norm. The spectral norm of an element of L only depends on its minimal polynomial
over K, so for K ⊆ L ⊆ M are two extensions of K, the spectral norm on M restricts to the
spectral norm on L. This work can be used to uniquely extend the p-adic norm on ℚ_[p] to an
algebraic closure of ℚ_[p], for example.
Details #
We define the spectral value and the spectral norm. We prove the norm extension theorem
[S. Bosch, U. Güntzer, R. Remmert, Non-Archimedean Analysis (Theorem 3.2.1/2)]
[BGR84] : given a nonarchimedean normed field K and an algebraic
extension L/K, the spectral norm is a power-multiplicative K-algebra norm on L extending
the norm on K. All K-algebra automorphisms of L are isometries with respect to this norm.
If L/K is finite, we get a formula relating the spectral norm on L with any other
power-multiplicative norm on L extending the norm on K.
Moreover, we also prove the unique norm extension theorem: if K is a field complete with respect
to a nontrivial nonarchimedean multiplicative norm and L/K is an algebraic extension, then the
spectral norm on L is a nonarchimedean multiplicative norm, and any power-multiplicative
K-algebra norm on L coincides with the spectral norm. More over, if L/K is finite, then L
is a complete space. This result is S. Bosch, U. Güntzer, R. Remmert, Non-Archimedean Analysis
(Theorem 3.2.4/2).
As a prerequisite, we formalize the proof of S. Bosch, U. Güntzer, R. Remmert, Non-Archimedean Analysis (Proposition 3.1.2/1).
Main Definitions #
spectralValue: the spectral value of a polynomial inR[X].spectralNorm: the spectral norm|y|_spis the spectral value of the minimal polynomial ofy : LoverK.spectralAlgNorm: the spectral norm is aK-algebra norm onL.spectralMulAlgNorm: the spectral norm is a multiplicativeK-algebra norm onL.
Main Results #
norm_le_spectralNorm: iffis a power-multiplicativeK-algebra norm onL, thenfis bounded above byspectralNorm K L.spectralNorm_eq_of_equiv: theK-algebra automorphisms ofLare isometries with respect to the spectral norm.spectralNorm_eq_iSup_of_finiteDimensional_normal: ifL/Kis finite and normal, thenspectralNorm K L x = iSup (fun (σ : Gal(L/K)) ↦ f (σ x)).isPowMul_spectralNorm: the spectral norm is power-multiplicative.isNonarchimedean_spectralNorm: the spectral norm is nonarchimedean.spectralNorm_extends: the spectral norm extends the norm onK.spectralNorm_unique: any power-multiplicativeK-algebra norm onLcoincides with the spectral norm.spectralAlgNorm_mul: the spectral norm onLis multiplicative.spectralNorm.completeSpace: ifL/Kis finite dimensional, thenLis a complete space with respect to topology induced by the spectral norm.
References #
Tags #
spectral, spectral norm, spectral value, seminorm, norm, nonarchimedean
The function ℕ → ℝ sending n to ‖ p.coeff n ‖^(1/(p.natDegree - n : ℝ)), if
n < p.natDegree, or to 0 otherwise.
Equations
Instances For
The spectral value of a polynomial in R[X], where R is a seminormed ring. One motivation
for the spectral value: if the norm on R is nonarchimedean, and if a monic polynomial
splits into linear factors, then its spectral value is the norm of its largest root.
See max_norm_root_eq_spectralValue.
Equations
- spectralValue p = iSup (spectralValueTerms p)
Instances For
The range of spectralValue_terms p is a finite set.
The sequence spectralValue_terms p is bounded above.
The sequence spectralValue_terms p is nonnegative.
The spectral value of a polynomial is nonnegative.
The polynomial X - r has spectral value ‖ r ‖.
The polynomial X ^ n has spectral value 0.
The spectral value of p equals zero if and only if p is of the form X ^ n.
The spectral value of a monic polynomial P is less than or equal to one if and only
if all of its coefficients have norm less than or equal to 1.
The norm of any root of p is bounded by the spectral value of p. See
[S. Bosch, U. Güntzer, R. Remmert, Non-Archimedean Analysis (Proposition 3.1.2/1(1))]
[BGR84].
If f is a nonarchimedean, power-multiplicative K-algebra norm on L, then the spectral
value of a polynomial p : K[X] that decomposes into linear factors in L is equal to the
maximum of the norms of the roots. See S. Bosch, U. Güntzer, R. Remmert, Non-Archimedean Analysis
(Proposition 3.1.2/1(2)).
If L is an algebraic extension of a normed field K and y : L then the spectral norm
spectralNorm K y : ℝ of y (written |y|_sp in the textbooks) is the spectral value of the
minimal polynomial of y over K.
Equations
- spectralNorm K L y = spectralValue (minpoly K y)
Instances For
If L/E/K is a tower of fields, then the spectral norm of x : E equals its spectral norm
when regarding x as an element of L.
If L/E/K is a tower of fields, then the spectral norm of x : E when regarded as an element
of the normal closure of E equals its spectral norm when regarding x as an element of L.
If L/E/K is a tower of fields and x = algebraMap E L g, then the spectral norm
of g : E when regarded as an element of the normal closure of E equals the spectral norm
of x : L.
spectralNorm K L (0 : L) = 0.
spectralNorm K L y is nonnegative.
spectralNorm K L y is positive if y ≠ 0.
If spectralNorm K L x = 0, then x = 0.
If f is a power-multiplicative K-algebra norm on L, then f
is bounded above by spectralNorm K L.
The K-algebra automorphisms of L are isometries with respect to the spectral norm.
If L/K is finite and normal, then spectralNorm K L x = supr (λ (σ : Gal(L/K)), f (σ x)).
If L/K is finite and normal, then spectralNorm K L = invariantExtension K L.
If L/K is finite and normal, then spectralNorm K L is power-multiplicative.
See also the more general result isPowMul_spectralNorm.
The spectral norm is a K-algebra norm on L when L/K is finite and normal.
See also spectralAlgNorm for a more general construction.
Equations
- spectralAlgNorm_of_finiteDimensional_normal K L = { toFun := spectralNorm K L, map_zero' := ⋯, add_le' := ⋯, neg' := ⋯, mul_le' := ⋯, eq_zero_of_map_eq_zero' := ⋯, smul' := ⋯ }
Instances For
The spectral norm is nonarchimedean when L/K is finite and normal.
See also isNonarchimedean_spectralNorm for a more general result.
The spectral norm extends the norm on K when L/K is finite and normal.
See also spectralNorm_extends for a more general result.
If L/K is finite and normal, and f is a power-multiplicative K-algebra norm on L
extending the norm on K, then f = spectralNorm K L.
The spectral norm extends the norm on K.
spectralNorm K L (-y) = spectralNorm K L y .
The spectral norm is compatible with the action of K.
The spectral norm is submultiplicative.
The spectral norm is power-multiplicative.
The spectral norm is nonarchimedean.
The spectral norm is a K-algebra norm on L.
Equations
- spectralAlgNorm K L = { toFun := spectralNorm K L, map_zero' := ⋯, add_le' := ⋯, neg' := ⋯, mul_le' := ⋯, eq_zero_of_map_eq_zero' := ⋯, smul' := ⋯ }
Instances For
If K is a field complete with respect to a nontrivial nonarchimedean multiplicative norm and
L/K is an algebraic extension, then any power-multiplicative K-algebra norm on L coincides
with the spectral norm.
If K is a field complete with respect to a nontrivial nonarchimedean multiplicative norm and
L/K is an algebraic extension, then any multiplicative ring norm on L extending the norm on
K coincides with the spectral norm.
Given a nonzero x : L, and assuming that (spectralAlgNorm h_alg hna) 1 ≤ 1, this is
the real-valued function sending y ∈ L to the limit of (f (y * x^n))/((f x)^n),
regarded as an algebra norm.
Equations
- algNormFromConst h1 hx = { toRingNorm := normFromConst h1 ⋯ ⋯, smul' := ⋯ }
Instances For
If K is a field complete with respect to a nontrivial nonarchimedean multiplicative norm and
L/K is an algebraic extension, then the spectral norm on L is multiplicative.
The spectral norm is a multiplicative K-algebra norm on L.
Equations
- spectralMulAlgNorm K L = { toAddGroupSeminorm := (spectralAlgNorm K L).toAddGroupSeminorm, map_one' := ⋯, map_mul' := ⋯, eq_zero_of_map_eq_zero' := ⋯, smul' := ⋯ }
Instances For
L with the spectral norm is a NormedField.
Equations
- One or more equations did not get rendered due to their size.
Instances For
L with the spectral norm is a NontriviallyNormedField.
Equations
- spectralNorm.nontriviallyNormedField K L = { toNormedField := spectralNorm.normedField K L, non_trivial := ⋯ }
Instances For
L with the spectral norm is a normed_add_comm_group.
Equations
Instances For
L with the spectral norm is a seminormed_add_comm_group.
Equations
Instances For
L with the spectral norm is a normed_space over K.
Equations
- spectralNorm.normedSpace K L = { toModule := inferInstance, norm_smul_le := ⋯ }
Instances For
The metric space structure on L induced by the spectral norm.
Equations
Instances For
The uniform space structure on L induced by the spectral norm.
Equations
Instances For
If L/K is finite dimensional, then L is a complete space with respect to topology induced
by the spectral norm.
Given an algebraic tower of fields E/L/K and an element x : L whose minimal polynomial f
over K splits into linear factors over E, the degree(f)th power of the spectral norm of x,
considered as an element of E, is equal to the spectral norm of the product of the E-valued
roots of f.
For x : L with minimal polynomial f(X) := X^n + a_{n-1}X^{n-1} + ... + a_0 over K,
the spectral norm of x is equal to ‖a_0‖^(1/(degree(f(X)))).