Documentation

Mathlib.NumberTheory.NumberField.ClassNumber

Class numbers of number fields #

This file defines the class number of a number field as the (finite) cardinality of the class group of its ring of integers. It also proves some elementary results on the class number.

Main definitions #

The way this theorem should be used is to first compute ⌊(M K)⌋₊ and then to use fin_cases to deal with the finite number of primes p in the interval.

noncomputable def NumberField.classNumber (K : Type u_1) [Field K] [NumberField K] :

The class number of a number field is the (finite) cardinality of the class group.

Equations
Instances For

    The class number of a number field is 1 iff the ring of integers is a PID.

    Let K be a number field and let M K be the Minkowski bound of K (by definition it is (4 / π) ^ nrComplexPlaces K * ((finrank ℚ K)! / (finrank ℚ K) ^ (finrank ℚ K) * √|discr K|)). To show that 𝓞 K is a PID it is enough to show that, for all (natural) primes p ∈ Finset.Icc 1 ⌊(M K)⌋₊, all ideals P above p such that p ^ (span ({p}).inertiaDeg P) ≤ ⌊(M K)⌋₊ are principal. This is the standard technique to prove that 𝓞 K is principal, see [MS77], discussion after Theorem 37.

    The way this theorem should be used is to first compute ⌊(M K)⌋₊ and then to use fin_cases to deal with the finite number of primes p in the interval.