Ideal norms #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the absolute ideal norm ideal.abs_norm (I : ideal R) : ℕ
as the cardinality of
the quotient R ⧸ I
(setting it to 0 if the cardinality is infinite),
and the relative ideal norm ideal.span_norm R (I : ideal S) : ideal S
as the ideal spanned by
the norms of elements in I
.
Main definitions #
submodule.card_quot (S : submodule R M)
: the cardinality of the quotientM ⧸ S
, inℕ
. This maps⊥
to0
and⊤
to1
.ideal.abs_norm (I : ideal R)
: the absolute ideal norm, defined as the cardinality of the quotientR ⧸ I
, as a bundled monoid-with-zero homomorphism.ideal.span_norm R (I : ideal S)
: the ideal spanned by the norms of elements inI
. This is used to defineideal.rel_norm
.ideal.rel_norm R (I : ideal S)
: the relative ideal norm as a bundled monoid-with-zero morphism, defined as the ideal spanned by the norms of elements inI
.
Main results #
map_mul ideal.abs_norm
: multiplicativity of the ideal norm is bundled in the definition ofideal.abs_norm
ideal.nat_abs_det_basis_change
: the ideal norm is given by the determinant of the basis change matrixideal.abs_norm_span_singleton
: the ideal norm of a principal ideal is the norm of its generatormap_mul ideal.rel_norm
: multiplicativity of the relative ideal norm
The cardinality of (M ⧸ S)
, if (M ⧸ S)
is finite, and 0
otherwise.
This is used to define the absolute ideal norm ideal.abs_norm
.
Equations
Multiplicity of the ideal norm, for coprime ideals. This is essentially just a repackaging of the Chinese Remainder Theorem.
If the d
from ideal.exists_mul_add_mem_pow_succ
is unique, up to P
,
then so are the c
s, up to P ^ (i + 1)
.
Inspired by [Neukirch], proposition 6.1
If a ∈ P^i \ P^(i+1)
and c ∈ P^i
, then a * d + e = c
for e ∈ P^(i+1)
.
ideal.mul_add_mem_pow_succ_unique
shows the choice of d
is unique, up to P
.
Inspired by [Neukirch], proposition 6.1
The choice of d
in ideal.exists_mul_add_mem_pow_succ
is unique, up to P
.
Inspired by [Neukirch], proposition 6.1
Multiplicity of the ideal norm, for powers of prime ideals.
Multiplicativity of the ideal norm in number rings.
The absolute norm of the ideal I : ideal R
is the cardinality of the quotient R ⧸ I
.
Equations
- ideal.abs_norm = {to_fun := submodule.card_quot semiring.to_module, map_zero' := _, map_one' := _, map_mul' := _}
Let e : S ≃ I
be an additive isomorphism (therefore a ℤ
-linear equiv).
Then an alternative way to compute the norm of I
is given by taking the determinant of e
.
See nat_abs_det_basis_change
for a more familiar formulation of this result.
Let b
be a basis for S
over ℤ
and bI
a basis for I
over ℤ
of the same dimension.
Then an alternative way to compute the norm of I
is given by taking the determinant of bI
over b
.
ideal.span_norm R (I : ideal S)
is the ideal generated by mapping algebra.norm R
over I
.
See also ideal.rel_norm
.
Equations
- ideal.span_norm R I = ideal.span (⇑(algebra.norm R) '' ↑I)
This condition eq_bot_or_top
is equivalent to being a field.
However, span_norm_mul_of_field
is harder to apply since we'd need to upgrade a comm_ring R
instance to a field R
instance.
Multiplicativity of ideal.span_norm
. simp-normal form is map_mul (ideal.rel_norm R)
.
The relative norm ideal.rel_norm R (I : ideal S)
, where R
and S
are Dedekind domains,
and S
is an extension of R
that is finite and free as a module.
Equations
- ideal.rel_norm R = {to_fun := ideal.span_norm R _inst_3, map_zero' := _, map_one' := _, map_mul' := _}