Seminorms and Local Convexity #
This file defines absorbent sets, balanced sets, seminorms and the Minkowski functional.
An absorbent set is one that "surrounds" the origin. The idea is made precise by requiring that any point belongs to all large enough scalings of the set. This is the vector world analog of a topological neighborhood of the origin.
A balanced set is one that is everywhere around the origin. This means that a • s ⊆ s
for all a
of norm less than 1
.
A seminorm is a function to the reals which is positive-semidefinite, absolutely homogeneous, and subadditive. They are closely related to convex sets and a topological vector space is locally convex if and only if its topology is induced by a family of seminorms.
The Minkowski functional of a set s
is the function which associates each point to how much you
need to scale s
for x
to be inside it. When s
is symmetric, convex and absorbent, its gauge is
a seminorm. Reciprocally, any seminorm arises as the gauge of some set, namely its unit ball. This
induces the equivalence of seminorms and locally convex topological vector spaces.
Main declarations #
For a vector space over a normed field:
absorbent
: A sets
is absorbent if every point eventually belongs to all large scalings ofs
.balanced
: A sets
is balanced ifa • s ⊆ s
for alla
of norm less than1
.seminorm
: A function to the reals that is positive-semidefinite, absolutely homogeneous, and subadditive.norm_seminorm 𝕜 E
: The norm onE
as a seminorm.gauge
: Aka Minkowksi functional.gauge s x
is the least (actually, an infimum)r
such thatx ∈ r • s
.gauge_seminorm
: The Minkowski functional as a seminorm, whens
is symmetric, convex and absorbent.
References #
TODO #
Define and show equivalence of two notions of local convexity for a topological vector space over ℝ or ℂ: that it has a local base of balanced convex absorbent sets, and that it carries the initial topology induced by a family of seminorms.
Prove the properties of balanced and absorbent sets of a real vector space.
Tags #
absorbent, balanced, seminorm, Minkowski functional, gauge, locally convex, LCTVS
Set Properties #
Absorbent and balanced sets in a vector space over a normed field.
Scalar multiplication (by possibly different types) of a balanced set is monotone.
A balanced set absorbs itself.
Topological vector space #
Every neighbourhood of the origin is absorbent.
The union of {0}
with the interior of a balanced set is balanced.
The interior of a balanced set is balanced if it contains the origin.
The closure of a balanced set is balanced.
Seminorms #
- to_fun : E → ℝ
- smul' : ∀ (a : 𝕜) (x : E), self.to_fun (a • x) = ∥a∥ * self.to_fun x
- triangle' : ∀ (x y : E), self.to_fun (x + y) ≤ self.to_fun x + self.to_fun y
A seminorm on a vector space over a normed field is a function to the reals that is positive semidefinite, positive homogeneous, and subadditive.
Equations
- seminorm.fun_like = {coe := seminorm.to_fun _inst_3, coe_injective' := _}
Helper instance for when there's too many metavariables to apply to_fun.to_coe_fn
.
Equations
- seminorm.inhabited = {default := 0}
Any action on ℝ
which factors through ℝ≥0
applies to a seminorm.
Equations
- seminorm.add_monoid = function.injective.add_monoid_smul coe_fn seminorm.add_monoid._proof_2 seminorm.add_monoid._proof_3 seminorm.coe_add seminorm.add_monoid._proof_4
Equations
- seminorm.ordered_cancel_add_comm_monoid = {add := add_monoid.add seminorm.add_monoid, add_assoc := _, add_left_cancel := _, zero := add_monoid.zero seminorm.add_monoid, zero_add := _, add_zero := _, nsmul := has_scalar.smul seminorm.has_scalar, nsmul_zero' := _, nsmul_succ' := _, add_comm := _, le := ordered_cancel_add_comm_monoid.le (function.injective.ordered_cancel_add_comm_monoid coe_fn seminorm.ordered_cancel_add_comm_monoid._proof_9 seminorm.ordered_cancel_add_comm_monoid._proof_10 seminorm.coe_add), lt := ordered_cancel_add_comm_monoid.lt (function.injective.ordered_cancel_add_comm_monoid coe_fn seminorm.ordered_cancel_add_comm_monoid._proof_9 seminorm.ordered_cancel_add_comm_monoid._proof_10 seminorm.coe_add), le_refl := _, le_trans := _, lt_iff_le_not_le := _, le_antisymm := _, add_le_add_left := _, le_of_add_le_add_left := _}
Equations
- seminorm.mul_action = function.injective.mul_action coe_fn seminorm.mul_action._proof_1 seminorm.mul_action._proof_2
coe_fn
as an add_monoid_hom
. Helper definition for showing that seminorm 𝕜 E
is
a module.
Equations
- seminorm.coe_fn_add_monoid_hom 𝕜 E = {to_fun := coe_fn seminorm.has_coe_to_fun, map_zero' := _, map_add' := _}
Equations
- seminorm.distrib_mul_action = function.injective.distrib_mul_action (seminorm.coe_fn_add_monoid_hom 𝕜 E) _ seminorm.distrib_mul_action._proof_1
Equations
- seminorm.module = function.injective.module R (seminorm.coe_fn_add_monoid_hom 𝕜 E) _ seminorm.module._proof_1
Equations
- seminorm.partial_order = partial_order.lift coe_fn seminorm.partial_order._proof_1
Equations
- seminorm.semilattice_sup = function.injective.semilattice_sup coe_fn seminorm.semilattice_sup._proof_1 seminorm.coe_sup
Composition of a seminorm with a linear map is a seminorm.
The composition as an add_monoid_hom
.
Equations
- seminorm.order_bot = {bot := 0, bot_le := _}
Seminorm ball #
The ball of radius r
at x
with respect to seminorm p
is the set of elements y
with
p (y - x) <
r`.
Seminorm-balls at the origin are balanced.
Seminorm-balls at the origin are absorbent.
Seminorm-balls containing the origin are absorbent.
A seminorm is convex. Also see convex_on_norm
.
Seminorm-balls are convex.
The norm as a seminorm #
The norm of a seminormed group as a seminorm.
Equations
- norm_seminorm 𝕜 E = {to_fun := norm semi_normed_group.to_has_norm, smul' := _, triangle' := _}
Balls at the origin are absorbent.
Balls containing the origin are absorbent.
Balls at the origin are balanced.
Minkowksi functional #
The Minkowski functional. Given a set s
in a real vector space, gauge s
is the functional
which sends x : E
to the smallest r : ℝ
such that x
is in s
scaled by r
.
If the given subset is absorbent
then the set we take an infimum over in gauge
is nonempty,
which is useful for proving many properties about the gauge.
The gauge evaluated at 0
is always zero (mathematically this requires 0
to be in the set s
but, the real infimum of the empty set in Lean being defined as 0
, it holds unconditionally).
The gauge is always nonnegative.
In textbooks, this is the homogeneity of the Minkowksi functional.
Topology induced by a family of seminorms #
A filter basis for the neighborhood filter of 0.
The add_group_filter_basis
induced by the filter basis seminorm_basis_zero
.
Equations
The module_filter_basis
induced by the filter basis seminorm_basis_zero
.
Equations
The proposition that a linear map is bounded between spaces with families of seminorms.
- topology_eq_with_seminorms : t = (seminorm.seminorm_module_filter_basis p).topology
The proposition that the topology of E
is induced by a family of seminorms p
.
Instances
The topology of a normed_space 𝕜 E
is induced by the seminorm norm_seminorm 𝕜 E
.