mathlib3 documentation

analysis.normed.order.lattice

Normed lattice ordered groups #

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

Motivated by the theory of Banach Lattices, we then define normed_lattice_add_comm_group 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.

@[class]
structure has_solid_norm (α : Type u_1) [normed_add_comm_group α] [lattice α] :
Prop

Let α be an add_comm_group 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 of this typeclass
theorem norm_le_norm_of_abs_le_abs {α : Type u_1} [normed_add_comm_group α] [lattice α] [has_solid_norm α] {a b : α} (h : |a| |b|) :

If α has a solid norm, then the balls centered at the origin of α are solid sets.

@[protected, instance]
@[protected, instance]
@[class]
structure normed_lattice_add_comm_group (α : Type u_1) :
Type u_1

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.

Instances of this typeclass
Instances of other typeclasses for normed_lattice_add_comm_group
  • normed_lattice_add_comm_group.has_sizeof_inst
theorem dual_solid {α : Type u_1} [normed_lattice_add_comm_group α] (a b : α) (h : b -b a -a) :
theorem norm_inf_sub_inf_le_add_norm {α : Type u_1} [normed_lattice_add_comm_group α] (a b c d : α) :
a b - c d a - c + b - d
theorem norm_sup_sub_sup_le_add_norm {α : Type u_1} [normed_lattice_add_comm_group α] (a b c d : α) :
a b - c d a - c + b - d
theorem norm_inf_le_add {α : Type u_1} [normed_lattice_add_comm_group α] (x y : α) :
theorem norm_sup_le_add {α : Type u_1} [normed_lattice_add_comm_group α] (x y : α) :
@[protected, instance]

Let α be a normed lattice ordered group. Then the infimum is jointly continuous.

@[protected, instance]

Let α be a normed lattice ordered group. Then α is a topological lattice in the norm topology.

Equations
theorem norm_abs_sub_abs {α : Type u_1} [normed_lattice_add_comm_group α] (a b : α) :
theorem norm_sup_sub_sup_le_norm {α : Type u_1} [normed_lattice_add_comm_group α] (x y z : α) :
x z - y z x - y
theorem norm_inf_sub_inf_le_norm {α : Type u_1} [normed_lattice_add_comm_group α] (x y z : α) :
x z - y z x - y
theorem lipschitz_with_sup_right {α : Type u_1} [normed_lattice_add_comm_group α] (z : α) :
lipschitz_with 1 (λ (x : α), x z)
theorem is_closed_nonneg {E : Type u_1} [normed_lattice_add_comm_group E] :
is_closed {x : E | 0 x}