Ideal norms #
This file defines the absolute ideal norm Ideal.absNorm (I : Ideal R) : ℕ
as the cardinality of
the quotient R ⧸ I
(setting it to 0 if the cardinality is infinite).
Main definitions #
Submodule.cardQuot (S : Submodule R M)
: the cardinality of the quotientM ⧸ S
, inℕ
. This maps⊥
to0
and⊤
to1
.Ideal.absNorm (I : Ideal R)
: the absolute ideal norm, defined as the cardinality of the quotientR ⧸ I
, as a bundled monoid-with-zero homomorphism.
Main results #
map_mul Ideal.absNorm
: multiplicativity of the ideal norm is bundled in the definition ofIdeal.absNorm
Ideal.natAbs_det_basis_change
: the ideal norm is given by the determinant of the basis change matrixIdeal.absNorm_span_singleton
: the ideal norm of a principal ideal is the norm of its generator
The cardinality of (M ⧸ S)
, if (M ⧸ S)
is finite, and 0
otherwise.
This is used to define the absolute ideal norm Ideal.absNorm
.
Equations
- S.cardQuot = S.toAddSubgroup.index
Instances For
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.absNorm = { toFun := Submodule.cardQuot, map_zero' := ⋯, map_one' := ⋯, map_mul' := ⋯ }
Instances For
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 natAbs_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
.