Convex bodies #
This file contains the definition of the type ConvexBody V
consisting of
convex, compact, nonempty subsets of a real topological vector space V
.
ConvexBody V
is a module over the nonnegative reals (NNReal
) and a pseudo-metric space.
If V
is a normed space, ConvexBody V
is a metric space.
TODO #
- define positive convex bodies, requiring the interior to be nonempty
- introduce support sets
- Characterise the interaction of the distance with algebraic operations, eg
dist (a • K) (a • L) = ‖a‖ * dist K L
,dist (a +ᵥ K) (a +ᵥ L) = dist K L
Tags #
convex, convex body
Let V
be a real topological vector space. A subset of V
is a convex body if and only if
it is convex, compact, and nonempty.
- carrier : Set V
The carrier set underlying a convex body: the set of points contained in it
A convex body has convex carrier set
- isCompact' : IsCompact self.carrier
A convex body has compact carrier set
- nonempty' : self.carrier.Nonempty
A convex body has non-empty carrier set
Instances For
Equations
- ConvexBody.instSetLike = { coe := ConvexBody.carrier, coe_injective' := ⋯ }
A convex body that is symmetric contains 0
.
Equations
- ConvexBody.instZero = { zero := { carrier := 0, convex' := ⋯, isCompact' := ⋯, nonempty' := ⋯ } }
Equations
- ConvexBody.instInhabited = { default := 0 }
Equations
- ConvexBody.instAdd = { add := fun (K L : ConvexBody V) => { carrier := ↑K + ↑L, convex' := ⋯, isCompact' := ⋯, nonempty' := ⋯ } }
Equations
- ConvexBody.instSMulNat = { smul := nsmulRec }
Equations
- ConvexBody.instAddMonoid = Function.Injective.addMonoid SetLike.coe ⋯ ⋯ ⋯ ⋯
Equations
- ConvexBody.instAddCommMonoid = Function.Injective.addCommMonoid SetLike.coe ⋯ ⋯ ⋯ ⋯
Equations
- ConvexBody.instSMulReal = { smul := fun (c : ℝ) (K : ConvexBody V) => { carrier := c • ↑K, convex' := ⋯, isCompact' := ⋯, nonempty' := ⋯ } }
Equations
- ConvexBody.instDistribMulActionReal = Function.Injective.distribMulAction { toFun := SetLike.coe, map_zero' := ⋯, map_add' := ⋯ } ⋯ ⋯
The convex bodies in a fixed space $V$ form a module over the nonnegative reals.
Convex bodies in a fixed seminormed space $V$ form a pseudo-metric space under the Hausdorff metric.
Equations
- One or more equations did not get rendered due to their size.
Let K
be a convex body that contains 0
and let u n
be a sequence of nonnegative real
numbers that tends to 0
. Then the intersection of the dilated bodies (1 + u n) • K
is equal
to K
.
Convex bodies in a fixed normed space V
form a metric space under the Hausdorff metric.
Equations
- ConvexBody.instMetricSpace = MetricSpace.mk ⋯