Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

[Merged by Bors] - feat(analysis/convex/uniform): Uniformly convex spaces #13480

Closed
wants to merge 7 commits into from

Conversation

YaelDillies
Copy link
Collaborator

@YaelDillies YaelDillies commented Apr 16, 2022

Define uniformly convex spaces and prove the implications inner_product_space ℝ E → uniform_convex_space E and uniform_convex_space E → strict_convex_space ℝ E.


Open in Gitpod

@YaelDillies YaelDillies added the awaiting-review The author would like community review of the PR label Apr 16, 2022
Comment on lines -1573 to -1588
/-- An inner product space is strictly convex. We do not register this as an instance for an inner
space over `𝕜`, `is_R_or_C 𝕜`, because there is no order of the typeclass argument that does not
lead to a search of `[is_scalar_tower ℝ ?m E]` with unknown `?m`. -/
instance inner_product_space.strict_convex_space : strict_convex_space ℝ F :=
begin
refine strict_convex_space.of_norm_add (λ x y h, _),
rw [same_ray_iff_norm_smul_eq, eq_comm, ← inner_eq_norm_mul_iff_real,
real_inner_eq_norm_add_mul_self_sub_norm_mul_self_sub_norm_mul_self_div_two, h,
add_mul_self_eq, sub_sub, add_sub_add_right_eq_sub, add_sub_cancel', mul_assoc,
mul_div_cancel_left],
exact _root_.two_ne_zero
end
Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

@urkud, do you wish to keep this proof around? Would it work to prove inner_product_space ℂ E → strict_convex_space ℂ E?

Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I don't want to talk about strict_convex_space ℂ E, so let's remove this proof. BTW, I have a better version of the lemma added in #13548 (I drop assumptions 0 < a and 0 < b; also, the proof is based on a more general fact about strict convex sets). It depends on #13631, #13656, and #13658.

Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Oh exciting! Ping me when it's out.

Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Let's merge your PR first.

@leanprover-community-bot-assistant leanprover-community-bot-assistant added merge-conflict Please `git merge origin/master` then a bot will remove this label. blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. and removed blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. labels Apr 19, 2022
@leanprover-community-bot-assistant leanprover-community-bot-assistant removed the merge-conflict Please `git merge origin/master` then a bot will remove this label. label Apr 22, 2022
@@ -172,6 +172,9 @@ lemma norm_add_le_of_le {g₁ g₂ : E} {n₁ n₂ : ℝ} (H₁ : ∥g₁∥ ≤
∥g₁ + g₂∥ ≤ n₁ + n₂ :=
le_trans (norm_add_le g₁ g₂) (add_le_add H₁ H₂)

lemma norm_add₃_le (x y z : E) : ∥x + y + z∥ ≤ ∥x∥ + ∥y∥ + ∥z∥ :=
Copy link
Member

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Cf. abs_add_three.

Copy link
Collaborator Author

@YaelDillies YaelDillies May 22, 2022

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Do you want me to rename this lemma? I think abs_add_three is a bad name because it looks like it's about |a + 3|.

variables [normed_space ℝ E]

lemma exists_forall_sphere_dist_add_le_two_mul_sub (hε : 0 < ε) (r : ℝ) :
∃ δ, 0 < δ ∧ ∀ ⦃x : E⦄, ∥x∥ = r → ∀ ⦃y⦄, ∥y∥ = r → ε ≤ ∥x - y∥ → ∥x + y∥ ≤ 2 * r - δ :=
Copy link
Member

@urkud urkud May 22, 2022

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

You don't use this lemma in the next one, so you can move it below exists_forall_ball_dist_add_le_two_mul_sub and easily deduce it from that lemma.

Copy link
Collaborator Author

@YaelDillies YaelDillies May 22, 2022

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Hmmm... yeah but actually once you use the modulus of convexity, this is really quite different.

Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I will delete it for now.

@urkud
Copy link
Member

urkud commented May 22, 2022

Thanks!
bors d+

@bors
Copy link

bors bot commented May 22, 2022

✌️ YaelDillies can now approve this pull request. To approve and merge a pull request, simply reply with bors r+. More detailed instructions are available here.

@github-actions github-actions bot added delegated The PR author may merge after reviewing final suggestions. and removed awaiting-review The author would like community review of the PR labels May 22, 2022
@YaelDillies
Copy link
Collaborator Author

Thanks! I will rework this with the modulus of convexity when I have time.

bors merge

bors bot pushed a commit that referenced this pull request May 22, 2022
Define uniformly convex spaces and prove the implications `inner_product_space ℝ E → uniform_convex_space E` and `uniform_convex_space E → strict_convex_space ℝ E`.
@bors
Copy link

bors bot commented May 22, 2022

Build failed (retrying...):

bors bot pushed a commit that referenced this pull request May 22, 2022
Define uniformly convex spaces and prove the implications `inner_product_space ℝ E → uniform_convex_space E` and `uniform_convex_space E → strict_convex_space ℝ E`.
@bors
Copy link

bors bot commented May 22, 2022

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(analysis/convex/uniform): Uniformly convex spaces [Merged by Bors] - feat(analysis/convex/uniform): Uniformly convex spaces May 22, 2022
@bors bors bot closed this May 22, 2022
@bors bors bot deleted the uniform_convex_space branch May 22, 2022 12:14
Ruben-VandeVelde added a commit that referenced this pull request Feb 3, 2023
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
delegated The PR author may merge after reviewing final suggestions.
Projects
None yet
Development

Successfully merging this pull request may close these issues.

4 participants