Normed lattice ordered groups #
Motivated by the theory of Banach Lattices, we then define NormedLatticeAddCommGroup
as a
lattice with a covariant normed group addition satisfying the solid axiom.
Main statements #
We show that a normed lattice ordered group is a topological lattice with respect to the norm topology.
References #
Tags #
normed, lattice, ordered, group
Normed lattice ordered groups #
Motivated by the theory of Banach Lattices, this section introduces normed lattice ordered groups.
Let α
be an AddCommGroup
with a Lattice
structure. A norm on α
is solid if, for a
and b
in α
, with absolute values |a|
and |b|
respectively, |a| ≤ |b|
implies ‖a‖ ≤ ‖b‖
.
Instances
If α
has a solid norm, then the balls centered at the origin of α
are solid sets.
Let α
be a normed commutative group equipped with a partial order covariant with addition, with
respect which α
forms a lattice. Suppose that α
is solid, that is to say, for a
and b
in
α
, with absolute values |a|
and |b|
respectively, |a| ≤ |b|
implies ‖a‖ ≤ ‖b‖
. Then α
is
said to be a normed lattice ordered group.
- add : α → α → α
- zero : α
- neg : α → α
- sub : α → α → α
- uniformity_dist : uniformity α = ⨅ (ε : ℝ), ⨅ (_ : ε > 0), Filter.principal {p : α × α | dist p.1 p.2 < ε}
- toBornology : Bornology α
- cobounded_sets : (Bornology.cobounded α).sets = {s : Set α | ∃ (C : ℝ), ∀ x ∈ sᶜ, ∀ y ∈ sᶜ, dist x y ≤ C}
- sup : α → α → α
- inf : α → α → α
Instances
A normed lattice ordered group is an ordered additive commutative group
Equations
- NormedLatticeAddCommGroup.toOrderedAddCommGroup = OrderedAddCommGroup.mk ⋯
Let α
be a normed lattice ordered group, then the order dual is also a
normed lattice ordered group.
Equations
- OrderDual.instNormedLatticeAddCommGroup = NormedLatticeAddCommGroup.mk ⋯
Let α
be a normed lattice ordered group. Then the infimum is jointly continuous.
Let α
be a normed lattice ordered group. Then α
is a topological lattice in the norm topology.