Zulip Chat Archive
Stream: maths
Topic: maximum modulus principle
Yury G. Kudryashov (Dec 25 2021 at 15:41):
Do we need some assumptions on the codomain of f : ℂ → E
to prove the maximum modulus principle? I can easily prove that
- if
is_max_on (norm ∘ f) (closed_ball c R) c
,R > 0
, thennorm ∘ f
is constant on this disc (+ corollaries); - if the norm on
E
is strictly convex, thenis_local_max (norm ∘ f) a
impliesf x = f a
neara
(+ corollaries).
Is the second statement true without the "strictly convex" assumption?
@Patrick Massot @Sebastien Gouezel @Heather Macbeth :up:
Yaël Dillies (Dec 25 2021 at 16:19):
Btw Yury I'm defining strictly convex spaces.
Sebastien Gouezel (Dec 25 2021 at 21:31):
You need some assumption. Let with the sup norm. Let . Then, for around , the norm of is constant equal to , and still is not constant.
Sebastien Gouezel (Dec 25 2021 at 21:32):
See https://www.ams.org/journals/proc/1967-018-04/S0002-9939-1967-0214794-2/ for instance.
Yury G. Kudryashov (Dec 26 2021 at 00:03):
For now, I'll formalize the weaker version and add a reference to this paper. Thanks!
Yury G. Kudryashov (Jan 19 2022 at 07:39):
@Yaël Dillies Do you have some draft? I have (some versions of the) strict Jensen inequality in #11552 and I would prefer to have a typeclass saying "norm is strictly convex".
Yury G. Kudryashov (Jan 19 2022 at 07:39):
With instances for complex
and (less urgent) Lp.
Yaël Dillies (Jan 19 2022 at 07:59):
We have (something close to) strict convexity of on branch#behrend. We use it in combinatorics!
Yaël Dillies (Jan 19 2022 at 08:01):
I haven't yet written the definition of strict_convex_space
because it is quite trivial from what we already have and I thought I would at least have the modulus of convexity on top to make it worth a PR, but if you need it now I can do it.
Yury G. Kudryashov (Jan 19 2022 at 08:07):
I just want to take "the norm is strictly convex" as a typeclass argument instead of an explicit one.
Yaël Dillies (Jan 19 2022 at 08:07):
Ah then wait a few minutes!
Yury G. Kudryashov (Jan 19 2022 at 08:08):
Thank you!
Yaël Dillies (Jan 19 2022 at 08:25):
Just to make sure, do we agree that a strictly convex space is a space where the norm is strictly convex? Because I never saw the equivalence with the fact that the unit ball is strictly convex.
Yaël Dillies (Jan 19 2022 at 08:45):
This really bugs me, because "strictly convex norm" refers to "the balls are strictly convex", not "the norm is a strictly convex function".
Yaël Dillies (Jan 19 2022 at 09:07):
Here are the two options
import analysis.convex.strict
import analysis.convex.topology
open metric set
class strict_convex_space_through_balls (𝕜 E : Type*) [normed_linear_ordered_field 𝕜]
[semi_normed_group E] [normed_space 𝕜 E] : Prop :=
(norm_strict_convex : strict_convex 𝕜 (ball (0 : E) 1))
class strict_convex_space_through_norm (E : Type*) [semi_normed_group E] [normed_space ℝ E] :
Prop :=
(norm_strict_convex : strict_convex_on ℝ univ (@norm E _))
lemma are_they_equivalent (E : Type*) [semi_normed_group E] [normed_space ℝ E] :
strict_convex_space_through_norm E ↔ strict_convex_space_through_balls ℝ E := sorry
The first one seems strictly convex more general?
Yury G. Kudryashov (Jan 19 2022 at 13:42):
Do you mean closed_ball
?
Yury G. Kudryashov (Jan 19 2022 at 13:54):
I shouldn't formalize things after midnight: clearly, norm
is not a strictly convex function on complex
(take x = 1
, y = 2
, any a
, b
)
Yury G. Kudryashov (Jan 19 2022 at 13:55):
So, I should redo the last theorem assuming that closed_ball 0 R
is convex.
Yaël Dillies (Jan 19 2022 at 14:22):
Yury G. Kudryashov said:
Do you mean
closed_ball
?
Uh, yes
Yaël Dillies (Jan 19 2022 at 14:23):
So the correct definition is the second one, right?
Yury G. Kudryashov (Jan 19 2022 at 15:21):
The correct definition is the first one with closed_ball
: strict_convex_space_through_norm
is never true on a non-trivial normed space (just take v
and v + v
).
Yury G. Kudryashov (Jan 19 2022 at 15:21):
(I'm not sure about radius 1 vs ∀ R
but they're equivalent for real
)
Yaël Dillies (Jan 19 2022 at 15:27):
That's what I meant :sweat_smile:
Yury G. Kudryashov (Jan 23 2022 at 17:02):
@Yaël Dillies Any news?
Yury G. Kudryashov (Jan 23 2022 at 17:03):
(if not, then I'll add a simple class with a couple of instances tonight)
Yaël Dillies (Jan 23 2022 at 17:07):
Yup, I have the stuff ready-ish if you need it.
Yury G. Kudryashov (Jan 23 2022 at 17:11):
PR?
Yaël Dillies (Jan 23 2022 at 17:12):
Will open it this evening.
Yury G. Kudryashov (Jan 30 2022 at 13:17):
Any news? @Yaël Dillies
Yaël Dillies (Jan 30 2022 at 22:24):
Just need to find an hour to put everything together.
Yury G. Kudryashov (Feb 02 2022 at 04:27):
Could you please open a PR with whatever you have on this subject?
Yury G. Kudryashov (Feb 02 2022 at 21:11):
@Yaël Dillies I'm sorry for poking you again but I would prefer if you either open a (possibly, not finalized) PR, or release the lock on this feature and let me implement it.
Yaël Dillies (Feb 02 2022 at 21:12):
Yes sorry, I've been having too much fun defining order categories. Doing it now.
Yaël Dillies (Feb 04 2022 at 16:58):
Are you happy with the PR?
Yury G. Kudryashov (Feb 04 2022 at 17:02):
I'll review it tonight. I'm trying to write a paper for ITP (deadline Feb. 8)
Yaël Dillies (Feb 04 2022 at 17:21):
Me too. Help :upside_down:
Yaël Dillies (Feb 18 2022 at 09:18):
@Yury G. Kudryashov, are you happy with the "two semirings" lemmas from #11794?
Yury G. Kudryashov (Apr 27 2022 at 02:15):
I'm trying to formalize a version of the maximum principle for strictly convex codomain.
Yury G. Kudryashov (Apr 27 2022 at 02:17):
I have the following problem: the completion of a strictly convex space may be not strictly convex. So, I have to either require [strict_convex_space F] [complete_space F]
or [strict_convex_space (completion F)]
.
Yury G. Kudryashov (Apr 27 2022 at 02:17):
Are there any better options?
Yury G. Kudryashov (Apr 27 2022 at 02:18):
E.g., I don't know whether the principle is true in a strictly convex space if the completion is not strictly convex.
Last updated: Dec 20 2023 at 11:08 UTC