mathlib3 documentation

analysis.convex.extreme

Extreme sets #

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

This file defines extreme sets and extreme points for sets in a module.

An extreme set of A is a subset of A that is as far as it can get in any outward direction: If point x is in it and point y ∈ A, then the line passing through x and y leaves A at x. This is an analytic notion of "being on the side of". It is weaker than being exposed (see is_exposed.is_extreme).

Main declarations #

Implementation notes #

The exact definition of extremeness has been carefully chosen so as to make as many lemmas unconditional (in particular, the Krein-Milman theorem doesn't need the set to be convex!). In practice, A is often assumed to be a convex set.

References #

See chapter 8 of Barry Simon, Convexity

TODO #

Prove lemmas relating extreme sets and points to the intrinsic frontier.

More not-yet-PRed stuff is available on the branch sperner_again.

def is_extreme (𝕜 : Type u_1) {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] (A B : set E) :
Prop

A set B is an extreme subset of A if B ⊆ A and all points of B only belong to open segments whose ends are in B.

Equations
Instances for is_extreme
def set.extreme_points (𝕜 : Type u_1) {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] (A : set E) :
set E

A point x is an extreme point of a set A if x belongs to no open segment with ends in A, except for the obvious open_segment x x.

Equations
@[protected, refl]
theorem is_extreme.refl (𝕜 : Type u_1) {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] (A : set E) :
is_extreme 𝕜 A A
@[protected]
theorem is_extreme.rfl {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} :
is_extreme 𝕜 A A
@[protected, trans]
theorem is_extreme.trans {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A B C : set E} (hAB : is_extreme 𝕜 A B) (hBC : is_extreme 𝕜 B C) :
is_extreme 𝕜 A C
@[protected]
theorem is_extreme.antisymm {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] :
@[protected, instance]
def is_extreme.is_partial_order {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] :
theorem is_extreme.inter {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A B C : set E} (hAB : is_extreme 𝕜 A B) (hAC : is_extreme 𝕜 A C) :
is_extreme 𝕜 A (B C)
@[protected]
theorem is_extreme.mono {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A B C : set E} (hAC : is_extreme 𝕜 A C) (hBA : B A) (hCB : C B) :
is_extreme 𝕜 B C
theorem is_extreme_Inter {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} {ι : Sort u_3} [nonempty ι] {F : ι set E} (hAF : (i : ι), is_extreme 𝕜 A (F i)) :
is_extreme 𝕜 A ( (i : ι), F i)
theorem is_extreme_bInter {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} {F : set (set E)} (hF : F.nonempty) (hA : (B : set E), B F is_extreme 𝕜 A B) :
is_extreme 𝕜 A ( (B : set E) (H : B F), B)
theorem is_extreme_sInter {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} {F : set (set E)} (hF : F.nonempty) (hAF : (B : set E), B F is_extreme 𝕜 A B) :
is_extreme 𝕜 A (⋂₀ F)
theorem mem_extreme_points {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} {x : E} :
x set.extreme_points 𝕜 A x A (x₁ : E), x₁ A (x₂ : E), x₂ A x open_segment 𝕜 x₁ x₂ x₁ = x x₂ = x
theorem mem_extreme_points_iff_extreme_singleton {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} {x : E} :
x set.extreme_points 𝕜 A is_extreme 𝕜 A {x}

x is an extreme point to A iff {x} is an extreme set of A.

theorem extreme_points_subset {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A : set E} :
@[simp]
theorem extreme_points_empty {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] :
@[simp]
theorem extreme_points_singleton {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {x : E} :
set.extreme_points 𝕜 {x} = {x}
theorem inter_extreme_points_subset_extreme_points_of_subset {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A B : set E} (hBA : B A) :
theorem is_extreme.extreme_points_subset_extreme_points {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A B : set E} (hAB : is_extreme 𝕜 A B) :
theorem is_extreme.extreme_points_eq {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_monoid E] [has_smul 𝕜 E] {A B : set E} (hAB : is_extreme 𝕜 A B) :
theorem is_extreme.convex_diff {𝕜 : Type u_1} {E : Type u_2} [ordered_semiring 𝕜] [add_comm_group E] [module 𝕜 E] {A B : set E} (hA : convex 𝕜 A) (hAB : is_extreme 𝕜 A B) :
convex 𝕜 (A \ B)
@[simp]
theorem extreme_points_prod {𝕜 : Type u_1} {E : Type u_2} {F : Type u_3} [ordered_semiring 𝕜] [add_comm_group E] [add_comm_group F] [module 𝕜 E] [module 𝕜 F] (s : set E) (t : set F) :
@[simp]
theorem extreme_points_pi {𝕜 : Type u_1} {ι : Type u_4} {π : ι Type u_5} [ordered_semiring 𝕜] [Π (i : ι), add_comm_group (π i)] [Π (i : ι), module 𝕜 (π i)] (s : Π (i : ι), set (π i)) :
set.extreme_points 𝕜 (set.univ.pi s) = set.univ.pi (λ (i : ι), set.extreme_points 𝕜 (s i))
theorem mem_extreme_points_iff_forall_segment {𝕜 : Type u_1} {E : Type u_2} [linear_ordered_ring 𝕜] [add_comm_group E] [module 𝕜 E] [densely_ordered 𝕜] [no_zero_smul_divisors 𝕜 E] {A : set E} {x : E} :
x set.extreme_points 𝕜 A x A (x₁ : E), x₁ A (x₂ : E), x₂ A x segment 𝕜 x₁ x₂ x₁ = x x₂ = x

A useful restatement using segment: x is an extreme point iff the only (closed) segments that contain it are those with x as one of their endpoints.

theorem convex.mem_extreme_points_iff_convex_diff {𝕜 : Type u_1} {E : Type u_2} [linear_ordered_ring 𝕜] [add_comm_group E] [module 𝕜 E] [densely_ordered 𝕜] [no_zero_smul_divisors 𝕜 E] {A : set E} {x : E} (hA : convex 𝕜 A) :
x set.extreme_points 𝕜 A x A convex 𝕜 (A \ {x})
theorem convex.mem_extreme_points_iff_mem_diff_convex_hull_diff {𝕜 : Type u_1} {E : Type u_2} [linear_ordered_ring 𝕜] [add_comm_group E] [module 𝕜 E] [densely_ordered 𝕜] [no_zero_smul_divisors 𝕜 E] {A : set E} {x : E} (hA : convex 𝕜 A) :
x set.extreme_points 𝕜 A x A \ (convex_hull 𝕜) (A \ {x})
theorem extreme_points_convex_hull_subset {𝕜 : Type u_1} {E : Type u_2} [linear_ordered_ring 𝕜] [add_comm_group E] [module 𝕜 E] [densely_ordered 𝕜] [no_zero_smul_divisors 𝕜 E] {A : set E} :