Zulip Chat Archive

Stream: mathlib4

Topic: how to prove the convex here.


Katherine Wei (May 15 2024 at 20:27):

theorem K_polar_convex: Convex  (K_polar vmatrix) := by
  rw[Convex]
  intro x hx
  rw[K_polar] at hx
  simp at hx

StarConvex ℝ x (K_polar vmatrix)

Ruben Van de Velde (May 15 2024 at 20:28):

Kinda hard to say without knowing what K_polar is

Katherine Wei (May 15 2024 at 20:28):

def K_polar: Set (Fin n  ) :=
{y |  x  K vmatrix, y ⬝ᵥ x  0}

Kim Morrison (May 15 2024 at 23:51):

(Posting questions as an #mwe makes it much more likely to get a good answer!)


Last updated: May 02 2025 at 03:31 UTC