Nonarchimedean functions #
A function f : α → R
is nonarchimedean if it satisfies the strong triangle inequality
f (a + b) ≤ max (f a) (f b)
for all a b : α
. This file proves basic properties of
nonarchimedean functions.
A nonnegative nonarchimedean function satisfies the triangle inequality.
If f
is a nonegative nonarchimedean function α → R
such that f 0 = 0
, then for every
n : ℕ
and a : α
, we have f (n • a) ≤ (f a)
.
If f
is a nonegative nonarchimedean function α → R
such that f 0 = 0
, then for every
n : ℕ
and a : α
, we have f (n * a) ≤ (f a)
.
If f
is a nonarchimedean additive group seminorm on α
with f 1 = 1
, then for every n : ℤ
we have f n ≤ 1
.
If f
is a nonarchimedean additive group seminorm on α
and x y : α
are such that
f x ≠ f y
, then f (x + y) = max (f x) (f y)
.
Given a nonarchimedean function α → R
, a function g : β → α
and a nonempty multiset
s : Multiset β
, we can always find b : β
belonging to s
such that
f (t.sum g) ≤ f (g b)
.
Given a nonarchimedean function α → R
, a function g : β → α
and a nonempty finset
t : Finset β
, we can always find b : β
belonging to t
such that f (t.sum g) ≤ f (g b)
.
Given a nonegative nonarchimedean function α → R
such that f 0 = 0
, a function g : β → α
and a multiset s : Multiset β
, we can always find b : β
, belonging to s
if s
is nonempty,
such that f (s.sum g) ≤ f (g b)
.
Given a nonegative nonarchimedean function α → R
such that f 0 = 0
, a function g : β → α
and a finset t : Finset β
, we can always find b : β
, belonging to t
if t
is nonempty,
such that f (t.sum g) ≤ f (g b)
.
Ultrametric inequality with Finset.Sum
.
If f
is a nonarchimedean additive group seminorm on a commutative ring α
, n : ℕ
, and
a b : α
, then we can find m : ℕ
such that m ≤ n
and
f ((a + b) ^ n) ≤ (f (a ^ m)) * (f (b ^ (n - m)))
.