Topological properties of convex sets #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We prove the following facts:
convex.interior: interior of a convex set is convex;convex.closure: closure of a convex set is convex;set.finite.compact_convex_hull: convex hull of a finite set is compact;set.finite.is_closed_convex_hull: convex hull of a finite set is closed.
Alias of the reverse direction of real.convex_iff_is_preconnected.
Standard simplex #
Every vector in std_simplex 𝕜 ι has max-norm at most 1.
std_simplex ℝ ι is bounded.
std_simplex ℝ ι is closed.
std_simplex ℝ ι is compact.
Topological vector space #
If s is a convex set, then a • interior s + b • closure s ⊆ interior s for all 0 < a,
0 ≤ b, a + b = 1. See also convex.combo_interior_self_subset_interior for a weaker version.
If s is a convex set, then a • interior s + b • s ⊆ interior s for all 0 < a, 0 ≤ b,
a + b = 1. See also convex.combo_interior_closure_subset_interior for a stronger version.
If s is a convex set, then a • closure s + b • interior s ⊆ interior s for all 0 ≤ a,
0 < b, a + b = 1. See also convex.combo_self_interior_subset_interior for a weaker version.
If s is a convex set, then a • s + b • interior s ⊆ interior s for all 0 ≤ a, 0 < b,
a + b = 1. See also convex.combo_closure_interior_subset_interior for a stronger version.
If x ∈ closure s and y ∈ interior s, then the segment (x, y] is included in interior s.
If x ∈ s and y ∈ interior s, then the segment (x, y] is included in interior s.
If x ∈ closure s and x + y ∈ interior s, then x + t y ∈ interior s for t ∈ (0, 1].
If x ∈ s and x + y ∈ interior s, then x + t y ∈ interior s for t ∈ (0, 1].
In a topological vector space, the interior of a convex set is convex.
In a topological vector space, the closure of a convex set is convex.
A convex set s is strictly convex provided that for any two distinct points of
s \ interior s, the line passing through these points has nonempty intersection with
interior s.
A convex set s is strictly convex provided that for any two distinct points x, y of
s \ interior s, the segment with endpoints x, y has nonempty intersection with
interior s.
Convex hull of a finite set is compact.
Convex hull of a finite set is closed.
If we dilate the interior of a convex set about a point in its interior by a scale t > 1,
the result includes the closure of the original set.
TODO Generalise this from convex sets to sets that are balanced / star-shaped about x.
If we dilate a convex set about a point in its interior by a scale t > 1, the interior of
the result includes the closure of the original set.
TODO Generalise this from convex sets to sets that are balanced / star-shaped about x.
If we dilate a convex set about a point in its interior by a scale t > 1, the interior of
the result includes the closure of the original set.
TODO Generalise this from convex sets to sets that are balanced / star-shaped about x.
A nonempty convex set is path connected.
A nonempty convex set is connected.
A convex set is preconnected.
Every topological vector space over ℝ is path connected.
Not an instance, because it creates enormous TC subproblems (turn on pp.all).