Convex sets and functions in vector spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In a 𝕜-vector space, we define the following objects and properties.
convex 𝕜 s
: A sets
is convex if for any two pointsx y ∈ s
it includessegment 𝕜 x y
.std_simplex 𝕜 ι
: The standard simplex inι → 𝕜
(currently requiresfintype ι
). It is the intersection of the positive quadrant with the hyperplanes.sum = 1
.
We also provide various equivalent versions of the definitions above, prove that some specific sets are convex.
TODO #
Generalize all this file to affine spaces.
Convexity of sets #
Convexity of sets.
The convex sets form an additive submonoid under pointwise addition.
The translation of a convex set is also convex.
The translation of a convex set is also convex.
Affine subspaces are convex.
The preimage of a convex set under an affine map is convex.
The image of a convex set under an affine map is convex.
Alternative definition of set convexity, using division.
Alias of the forward direction of convex_iff_ord_connected
.
Convexity of submodules/subspaces #
Simplex #
The standard simplex in the space of functions ι → 𝕜
is the set of vectors with non-negative
coordinates with total sum 1
. This is the free object in the category of convex spaces.
Equations
- std_simplex 𝕜 ι = {f : ι → 𝕜 | (∀ (x : ι), 0 ≤ f x) ∧ finset.univ.sum (λ (x : ι), f x) = 1}