Zulip Chat Archive

Stream: maths

Topic: strict convexity


Yaรซl Dillies (Sep 29 2021 at 17:03):

Can we define strict convexity without a topology? The definition on wikipedia is

import analysis.convex.basic
import topology.basic

def strict_convex {๐•œ E : Type*} [ordered_semiring ๐•œ] [add_comm_monoid E] [topological_space E]
  [has_scalar ๐•œ E] (s : set E) : Prop :=
โˆ€ x y, open_segment ๐•œ x y โŠ† interior s

Yaรซl Dillies (Sep 29 2021 at 17:08):

I'm thinking of

def strict_convex {๐•œ E : Type*} [ordered_semiring ๐•œ] [add_comm_group E] [has_scalar ๐•œ E]
  (s : set E) : Prop :=
โˆ€ t, is_extreme ๐•œ s t โ†’ โˆ€ x y : E, x โ‰  y โ†’ โˆ€ z, z โˆˆ open_segment ๐•œ x y โ†’ z โˆˆ t โ†’ t = s

Yaรซl Dillies (Sep 29 2021 at 17:09):

which should be read as "There's no plane on the surface of the set"

Reid Barton (Sep 29 2021 at 17:32):

Is that missing some parentheses?

Yaรซl Dillies (Sep 29 2021 at 18:03):

Hmm, no?

Yaรซl Dillies (Sep 29 2021 at 18:10):

Here's a maybe cleaner way to write my proposed definition:

def strict_convex {๐•œ E : Type*} [ordered_semiring ๐•œ] [add_comm_group E] [has_scalar ๐•œ E]
  (s : set E) : Prop :=
โˆ€ t, is_extreme ๐•œ s t โ†’ โˆ€ x, x โˆˆ t โ†’ x โˆ‰ s.extreme_points ๐•œ โ†’ t = s

Eric Wieser (Sep 29 2021 at 18:22):

That's the same as this definition, right?

โˆ€ t, is_extreme ๐•œ s t โ†’ (t \ s.extreme_points ๐•œ).nonempty โ†’ t = s

Yaรซl Dillies (Sep 29 2021 at 19:36):

Yup, because of the elimination rule for โˆƒ.

Eric Wieser (Sep 29 2021 at 19:54):

Which I guess you could also write as

โˆ€ t, is_extreme ๐•œ s t โ†’ ยฌ(t โŠ† s.extreme_points ๐•œ) โ†’ t = s

David Wรคrn (Sep 29 2021 at 20:34):

is x โˆˆ interior s different from โˆ€ v, โˆƒ r > 0, x + r โ€ข v โˆˆ s at the intended level of generality?

Yaรซl Dillies (Sep 29 2021 at 20:36):

Oh yeah. Take a union of infinitely many concentric spheres

Yaรซl Dillies (Sep 29 2021 at 20:37):

My above proposed definitions don't imply convex ๐•œ s... Maybe we can just add convex ๐•œ s โˆง?

David Wรคrn (Sep 29 2021 at 21:01):

I think I wanted to say โˆ€ v, โˆƒ r > 0, โˆ€ t โˆˆ Icc 0 r, x + t โ€ข v โˆˆ s

Yaรซl Dillies (Oct 01 2021 at 12:28):

Ahah! I think I got the idea.

Yaรซl Dillies (Oct 01 2021 at 12:30):

What you want is to not have any planar bits on the boundary. So what you can ask for is that any nonzero linear functional reaches a single maximum.

Yaรซl Dillies (Oct 01 2021 at 12:31):

which can be rewritten (thanks to someone's API :innocent:) as โˆ€ t, is_exposed ๐•œ s t โ†’ ยฌ s โŠ† t โ†’ t.subsingleton.

Yaรซl Dillies (Oct 02 2021 at 14:04):

The problem with the above definition is that it requires a normed space. I'm going to replace is_exposed with is_extreme.

Yaรซl Dillies (Oct 02 2021 at 14:05):

Note that the difference between the usual definition will then be that "flat" sets can be strictly convex, because the topology doesn't see them.

Yaรซl Dillies (Oct 02 2021 at 14:06):

Does anyone know whether that'll make a difference in applications?


Last updated: Dec 20 2023 at 11:08 UTC