Admissible absolute values on polynomials #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines an admissible absolute value polynomial.card_pow_degree_is_admissible
which we
use to show the class number of the ring of integers of a function field is finite.
Main results #
polynomial.card_pow_degree_is_admissible
showscard_pow_degree
, mappingp : polynomial 𝔽_q
toq ^ degree p
, is admissible
If A
is a family of enough low-degree polynomials over a finite semiring, there is a
pair of equal elements in A
.
If A
is a family of enough low-degree polynomials over a finite ring,
there is a pair of elements in A
(with different indices but not necessarily
distinct), such that their difference has small degree.
If A
is a family of enough low-degree polynomials over a finite field,
there is a pair of elements in A
(with different indices but not necessarily
distinct), such that the difference of their remainders is close together.
If x
is close to y
and y
is close to z
, then x
and z
are at least as close.
A slightly stronger version of exists_partition
on which we perform induction on n
:
for all ε > 0
, we can partition the remainders of any family of polynomials A
into equivalence classes, where the equivalence(!) relation is "closer than ε
".
For all ε > 0
, we can partition the remainders of any family of polynomials A
into classes, where all remainders in a class are close together.
λ p, fintype.card Fq ^ degree p
is an admissible absolute value.
We set q ^ degree 0 = 0
.
Equations
- polynomial.card_pow_degree_is_admissible = {to_is_euclidean := _, card := λ (ε : ℝ), fintype.card Fq ^ ⌈-real.log ε / real.log ↑(fintype.card Fq)⌉₊, exists_partition' := _}