Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2022-08-21 19:16 0da54467

View on Github →

refactor(analysis/convex/basic): Redefine convexity in terms of star-convexity (#16173) Change the definition from

def convex : Prop :=
∀ ⦃x y : E⦄, x ∈ s → y ∈ s → ∀ ⦃a b : 𝕜⦄, 0 ≤ a → 0 ≤ b → a + b = 1 →
  a • x + b • y ∈ s

to

def convex : Prop := ∀ ⦃x : E⦄, x ∈ s → star_convex 𝕜 x s

which is defeq up to swapping the second and third foralls. This allows golfing the convex API in terms of the star_convex one. Also generalize convex_pi by limiting quantification to the set.

Estimated changes

deleted theorem convex.combo_affine_apply
deleted theorem convex.combo_eq_vadd
modified theorem convex.prod
added theorem convex.star_convex
added theorem convex.star_convex_iff
modified def convex
modified theorem convex_empty
modified theorem convex_iff_segment_subset
modified theorem convex_univ
deleted theorem submodule.convex
deleted theorem subspace.convex