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 : α
- nsmul_zero : ∀ (x : α), AddMonoid.nsmul 0 x = 0
- nsmul_succ : ∀ (n : ℕ) (x : α), AddMonoid.nsmul (n + 1) x = AddMonoid.nsmul n x + x
- neg : α → α
- sub : α → α → α
- sub_eq_add_neg : ∀ (a b : α), a - b = a + -b
- zsmul_zero' : ∀ (a : α), SubNegMonoid.zsmul 0 a = 0
- zsmul_succ' : ∀ (n : ℕ) (a : α), SubNegMonoid.zsmul (↑n.succ) a = SubNegMonoid.zsmul (↑n) a + a
- zsmul_neg' : ∀ (n : ℕ) (a : α), SubNegMonoid.zsmul (Int.negSucc n) a = -SubNegMonoid.zsmul (↑n.succ) a
- neg_add_cancel : ∀ (a : α), -a + a = 0
- edist_dist : ∀ (x y : α), PseudoMetricSpace.edist x y = ENNReal.ofReal (dist x y)
- 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}
- eq_of_dist_eq_zero : ∀ {x y : α}, dist x y = 0 → x = y
- le_antisymm : ∀ (a b : α), a ≤ b → b ≤ a → a = b
- sup : α → α → α
- le_sup_left : ∀ (a b : α), a ≤ SemilatticeSup.sup a b
- le_sup_right : ∀ (a b : α), b ≤ SemilatticeSup.sup a b
- sup_le : ∀ (a b c : α), a ≤ c → b ≤ c → SemilatticeSup.sup a b ≤ c
- inf : α → α → α
- inf_le_left : ∀ (a b : α), Lattice.inf a b ≤ a
- inf_le_right : ∀ (a b : α), Lattice.inf a b ≤ b
- le_inf : ∀ (a b c : α), a ≤ b → a ≤ c → a ≤ Lattice.inf b c
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.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Let α
be a normed lattice ordered group. Then α
is a topological lattice in the norm topology.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯