Seminorms and norms on rings #
This file defines seminorms and norms on rings. These definitions are useful when one needs to consider multiple (semi)norms on a given ring.
Main declarations #
For a ring R
:
RingSeminorm
: A seminorm on a ringR
is a functionf : R → ℝ
that preserves zero, takes nonnegative values, is subadditive and submultiplicative and such thatf (-x) = f x
for allx ∈ R
.RingNorm
: A seminormf
is a norm iff x = 0
if and only ifx = 0
.MulRingSeminorm
: A multiplicative seminorm on a ringR
is a ring seminorm that preserves multiplication.MulRingNorm
: A multiplicative norm on a ringR
is a ring norm that preserves multiplication.
Notes #
The corresponding hom classes are defined in Mathlib.Analysis.Order.Hom.Basic
to be used by
absolute values.
References #
- [S. Bosch, U. Güntzer, R. Remmert, Non-Archimedean Analysis][bosch-guntzer-remmert]
Tags #
ring_seminorm, ring_norm
- toFun : R → ℝ
- map_zero' : AddGroupSeminorm.toFun s.toAddGroupSeminorm 0 = 0
- add_le' : ∀ (r s_1 : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (r + s_1) ≤ AddGroupSeminorm.toFun s.toAddGroupSeminorm r + AddGroupSeminorm.toFun s.toAddGroupSeminorm s_1
- neg' : ∀ (r : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (-r) = AddGroupSeminorm.toFun s.toAddGroupSeminorm r
- mul_le' : ∀ (x y : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (x * y) ≤ AddGroupSeminorm.toFun s.toAddGroupSeminorm x * AddGroupSeminorm.toFun s.toAddGroupSeminorm y
The property of a
RingSeminorm
that for allx
andy
in the ring, the norm ofx * y
is less than the norm ofx
times the norm ofy
.
A seminorm on a ring R
is a function f : R → ℝ
that preserves zero, takes nonnegative
values, is subadditive and submultiplicative and such that f (-x) = f x
for all x ∈ R
.
Instances For
- toFun : R → ℝ
- map_zero' : AddGroupSeminorm.toFun s.toAddGroupSeminorm 0 = 0
- add_le' : ∀ (r s_1 : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (r + s_1) ≤ AddGroupSeminorm.toFun s.toAddGroupSeminorm r + AddGroupSeminorm.toFun s.toAddGroupSeminorm s_1
- neg' : ∀ (r : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (-r) = AddGroupSeminorm.toFun s.toAddGroupSeminorm r
- mul_le' : ∀ (x y : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (x * y) ≤ AddGroupSeminorm.toFun s.toAddGroupSeminorm x * AddGroupSeminorm.toFun s.toAddGroupSeminorm y
- eq_zero_of_map_eq_zero' : ∀ (x : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm x = 0 → x = 0
If the image under the seminorm is zero, then the argument is zero.
A function f : R → ℝ
is a norm on a (nonunital) ring if it is a seminorm and f x = 0
implies x = 0
.
Instances For
- toFun : R → ℝ
- map_zero' : AddGroupSeminorm.toFun s.toAddGroupSeminorm 0 = 0
- add_le' : ∀ (r s_1 : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (r + s_1) ≤ AddGroupSeminorm.toFun s.toAddGroupSeminorm r + AddGroupSeminorm.toFun s.toAddGroupSeminorm s_1
- neg' : ∀ (r : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (-r) = AddGroupSeminorm.toFun s.toAddGroupSeminorm r
- map_one' : AddGroupSeminorm.toFun s.toAddGroupSeminorm 1 = 1
The proposition that the function preserves 1
- map_mul' : ∀ (x y : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (x * y) = AddGroupSeminorm.toFun s.toAddGroupSeminorm x * AddGroupSeminorm.toFun s.toAddGroupSeminorm y
The proposition that the function preserves multiplication
A multiplicative seminorm on a ring R
is a function f : R → ℝ
that preserves zero and
multiplication, takes nonnegative values, is subadditive and such that f (-x) = f x
for all x
.
Instances For
- toFun : R → ℝ
- map_zero' : AddGroupSeminorm.toFun s.toAddGroupSeminorm 0 = 0
- add_le' : ∀ (r s_1 : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (r + s_1) ≤ AddGroupSeminorm.toFun s.toAddGroupSeminorm r + AddGroupSeminorm.toFun s.toAddGroupSeminorm s_1
- neg' : ∀ (r : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (-r) = AddGroupSeminorm.toFun s.toAddGroupSeminorm r
- map_one' : AddGroupSeminorm.toFun s.toAddGroupSeminorm 1 = 1
- map_mul' : ∀ (x y : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm (x * y) = AddGroupSeminorm.toFun s.toAddGroupSeminorm x * AddGroupSeminorm.toFun s.toAddGroupSeminorm y
- eq_zero_of_map_eq_zero' : ∀ (x : R), AddGroupSeminorm.toFun s.toAddGroupSeminorm x = 0 → x = 0
If the image under the seminorm is zero, then the argument is zero.
A multiplicative norm on a ring R
is a multiplicative ring seminorm such that f x = 0
implies x = 0
.
Instances For
Helper instance for when there's too many metavariables to apply FunLike.hasCoeToFun
.
The trivial seminorm on a ring R
is the RingSeminorm
taking value 0
at 0
and 1
at
every other element.
The norm of a NonUnitalSeminormedRing
as a RingSeminorm
.
Instances For
Helper instance for when there's too many metavariables to apply FunLike.hasCoeToFun
.
The trivial norm on a ring R
is the RingNorm
taking value 0
at 0
and 1
at every
other element.
Helper instance for when there's too many metavariables to apply FunLike.hasCoeToFun
.
The trivial seminorm on a ring R
is the MulRingSeminorm
taking value 0
at 0
and 1
at
every other element.
Helper instance for when there's too many metavariables to apply FunLike.hasCoeToFun
.
The trivial norm on a ring R
is the MulRingNorm
taking value 0
at 0
and 1
at every
other element.
A nonzero ring seminorm on a field K
is a ring norm.
Instances For
The norm of a NonUnitalNormedRing
as a RingNorm
.