mathlib3 documentation

number_theory.padics.padic_norm

p-adic norm #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines the p-adic norm on .

The p-adic valuation on is the difference of the multiplicities of p in the numerator and denominator of q. This function obeys the standard properties of a valuation, with the appropriate assumptions on p.

The valuation induces a norm on . This norm is a nonarchimedean absolute value. It takes values in {0} ∪ {1/p^k | k ∈ ℤ}.

Notations #

This file uses the local notation /. for rat.mk.

Implementation notes #

Much, but not all, of this file assumes that p is prime. This assumption is inferred automatically by taking [fact p.prime] as a type class argument.

References #

Tags #

p-adic, p adic, padic, norm, valuation

def padic_norm (p : ) (q : ) :

If q ≠ 0, the p-adic norm of a rational q is p ^ -padic_val_rat p q. If q = 0, the p-adic norm of q is 0.

Equations
Instances for padic_norm
@[protected, simp]
theorem padic_norm.eq_zpow_of_nonzero {p : } {q : } (hq : q 0) :

Unfolds the definition of the p-adic norm of q when q ≠ 0.

@[protected]
theorem padic_norm.nonneg {p : } (q : ) :

The p-adic norm is nonnegative.

@[protected, simp]
theorem padic_norm.zero {p : } :

The p-adic norm of 0 is 0.

@[protected, simp]
theorem padic_norm.one {p : } :

The p-adic norm of 1 is 1.

theorem padic_norm.padic_norm_p {p : } (hp : 1 < p) :

The p-adic norm of p is p⁻¹ if p > 1.

See also padic_norm.padic_norm_p_of_prime for a version assuming p is prime.

@[simp]

The p-adic norm of p is p⁻¹ if p is prime.

See also padic_norm.padic_norm_p for a version assuming 1 < p.

theorem padic_norm.padic_norm_of_prime_of_ne {p q : } [p_prime : fact (nat.prime p)] [q_prime : fact (nat.prime q)] (neq : p q) :

The p-adic norm of q is 1 if q is prime and not equal to p.

theorem padic_norm.padic_norm_p_lt_one {p : } (hp : 1 < p) :

The p-adic norm of p is less than 1 if 1 < p.

See also padic_norm.padic_norm_p_lt_one_of_prime for a version assuming p is prime.

The p-adic norm of p is less than 1 if p is prime.

See also padic_norm.padic_norm_p_lt_one for a version assuming 1 < p.

@[protected]
theorem padic_norm.values_discrete {p : } {q : } (hq : q 0) :
(z : ), padic_norm p q = p ^ -z

padic_norm p q takes discrete values p ^ -z for z : ℤ.

@[protected, simp]
theorem padic_norm.neg {p : } (q : ) :

padic_norm p is symmetric.

@[protected]
theorem padic_norm.nonzero {p : } [hp : fact (nat.prime p)] {q : } (hq : q 0) :

If q ≠ 0, then padic_norm p q ≠ 0.

theorem padic_norm.zero_of_padic_norm_eq_zero {p : } [hp : fact (nat.prime p)] {q : } (h : padic_norm p q = 0) :
q = 0

If the p-adic norm of q is 0, then q is 0.

@[protected, simp]
theorem padic_norm.mul {p : } [hp : fact (nat.prime p)] (q r : ) :

The p-adic norm is multiplicative.

@[protected, simp]
theorem padic_norm.div {p : } [hp : fact (nat.prime p)] (q r : ) :

The p-adic norm respects division.

@[protected]
theorem padic_norm.of_int {p : } [hp : fact (nat.prime p)] (z : ) :

The p-adic norm of an integer is at most 1.

@[protected]
theorem padic_norm.nonarchimedean {p : } [hp : fact (nat.prime p)] {q r : } :

The p-adic norm is nonarchimedean: the norm of p + q is at most the max of the norm of p and the norm of q.

theorem padic_norm.triangle_ineq {p : } [hp : fact (nat.prime p)] (q r : ) :

The p-adic norm respects the triangle inequality: the norm of p + q is at most the norm of p plus the norm of q.

@[protected]
theorem padic_norm.sub {p : } [hp : fact (nat.prime p)] {q r : } :

The p-adic norm of a difference is at most the max of each component. Restates the archimedean property of the p-adic norm.

theorem padic_norm.add_eq_max_of_ne {p : } [hp : fact (nat.prime p)] {q r : } (hne : padic_norm p q padic_norm p r) :

If the p-adic norms of q and r are different, then the norm of q + r is equal to the max of the norms of q and r.

@[protected, instance]

The p-adic norm is an absolute value: positive-definite and multiplicative, satisfying the triangle inequality.

theorem padic_norm.dvd_iff_norm_le {p : } [hp : fact (nat.prime p)] {n : } {z : } :
theorem padic_norm.int_eq_one_iff {p : } [hp : fact (nat.prime p)] (m : ) :

The p-adic norm of an integer m is one iff p doesn't divide m.

theorem padic_norm.int_lt_one_iff {p : } [hp : fact (nat.prime p)] (m : ) :
theorem padic_norm.of_nat {p : } [hp : fact (nat.prime p)] (m : ) :
theorem padic_norm.nat_eq_one_iff {p : } [hp : fact (nat.prime p)] (m : ) :

The p-adic norm of a natural m is one iff p doesn't divide m.

theorem padic_norm.nat_lt_one_iff {p : } [hp : fact (nat.prime p)] (m : ) :
theorem padic_norm.sum_lt {p : } [hp : fact (nat.prime p)] {α : Type u_1} {F : α } {t : } {s : finset α} :
s.nonempty ( (i : α), i s padic_norm p (F i) < t) padic_norm p (s.sum (λ (i : α), F i)) < t
theorem padic_norm.sum_le {p : } [hp : fact (nat.prime p)] {α : Type u_1} {F : α } {t : } {s : finset α} :
s.nonempty ( (i : α), i s padic_norm p (F i) t) padic_norm p (s.sum (λ (i : α), F i)) t
theorem padic_norm.sum_lt' {p : } [hp : fact (nat.prime p)] {α : Type u_1} {F : α } {t : } {s : finset α} (hF : (i : α), i s padic_norm p (F i) < t) (ht : 0 < t) :
padic_norm p (s.sum (λ (i : α), F i)) < t
theorem padic_norm.sum_le' {p : } [hp : fact (nat.prime p)] {α : Type u_1} {F : α } {t : } {s : finset α} (hF : (i : α), i s padic_norm p (F i) t) (ht : 0 t) :
padic_norm p (s.sum (λ (i : α), F i)) t