Admissible absolute values #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4. This file defines a structure
absolute_value.is_admissiblewhich we use to show the class number of the ring of integers of a global field is finite.
Main definitions #
absolute_value.is_admissible abvstates the absolute valueabv : R → ℤrespects the Euclidean domain structure onR, and that a large enough set of elements ofR^ncontains a pair of elements whose remainders are pointwise close together.
Main results #
absolute_value.abs_is_admissibleshows the "standard" absolute value onℤ, mapping negativexto-x, is admissible.polynomial.card_pow_degree_is_admissibleshowscard_pow_degree, mappingp : polynomial 𝔽_qtoq ^ degree p, is admissible
- to_is_euclidean : abv.is_euclidean
- card : ℝ → ℕ
- exists_partition' : ∀ (n : ℕ) {ε : ℝ}, 0 < ε → ∀ {b : R}, b ≠ 0 → ∀ (A : fin n → R), ∃ (t : fin n → fin (self.card ε)), ∀ (i₀ i₁ : fin n), t i₀ = t i₁ → ↑(⇑abv (A i₁ % b - A i₀ % b)) < ⇑abv b • ε
An absolute value R → ℤ is admissible if it respects the Euclidean domain
structure and a large enough set of elements in R^n will contain a pair of
elements whose remainders are pointwise close together.
Instances for absolute_value.is_admissible
- absolute_value.is_admissible.has_sizeof_inst
- absolute_value.is_admissible.inhabited
For all ε > 0 and finite families A, we can partition the remainders of A mod b
into abv.card ε sets, such that all elements in each part of remainders are close together.
Any large enough family of vectors in R^n has a pair of elements
whose remainders are close together, pointwise.
Any large enough family of vectors in R^ι has a pair of elements
whose remainders are close together, pointwise.