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/normed_space/finite_dimension): Riesz theorem on compact unit ball and finite dimension #9147

Closed
wants to merge 4 commits into from

Conversation

sgouezel
Copy link
Collaborator


Open in Gitpod

@sgouezel sgouezel added the awaiting-review The author would like community review of the PR label Sep 11, 2021

/-- A sequence of points in an infinite-dimensional space, which are all bounded by `R` and at
distance at least `1`. Use `exists_seq_norm_le_le_norm_sub` instead. -/
noncomputable def exists_seq_norm_le_one_le_norm_sub_aux
Copy link
Member

Choose a reason for hiding this comment

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

Suggested change
noncomputable def exists_seq_norm_le_one_le_norm_sub_aux
noncomputable def seq_norm_le_one_le_norm_sub_aux

Should it be private?

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 think Floris told me that he hated private declarations because they can't be printed or checked, so I don't mark anything as private any more.

`exists_seq_norm_le_one_le_norm_sub`. -/
theorem exists_seq_norm_le_one_le_norm_sub' {c : 𝕜} (hc : 1 < ∥c∥) {R : ℝ} (hR : ∥c∥ < R)
(h : ¬ (finite_dimensional 𝕜 E)) :
∃ f : ℕ → E, (∀ n, ∥f n∥ ≤ R) ∧ (∀ m n, m ≠ n → 1 ≤ ∥f m - f n∥) :=
Copy link
Member

@urkud urkud Sep 11, 2021

Choose a reason for hiding this comment

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

I saw this kind of induction more than once. Should we have a lemma like this one?

lemma nat.exists_fun_forall_lt_imp {α : Type*} (p : α → Prop) (r : α → α → Prop)
  (H : ∀ (n : ℕ) (f : ℕ → α), ∃ y, p y ∧ ∀ k < n, r (f k) y) :
  ∃ f : ℕ → α, (∀ n, p n) ∧ ∀ m n, m < n → r m n := sorry

Copy link
Member

Choose a reason for hiding this comment

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

BTW, H can assume that f satisfies ∀ k < n, p (f k) and ∀ k l, k < l → l < n → r (f k) (f l).

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 have added a version expressed in terms of finsets: if for any finset s one can find a point y with r x y for all points in the finset, then one can find a sequence with r (f m) (f n) whenever m < n.

`exists_seq_norm_le_one_le_norm_sub`. -/
theorem exists_seq_norm_le_one_le_norm_sub' {c : 𝕜} (hc : 1 < ∥c∥) {R : ℝ} (hR : ∥c∥ < R)
(h : ¬ (finite_dimensional 𝕜 E)) :
∃ f : ℕ → E, (∀ n, ∥f n∥ ≤ R) ∧ (∀ m n, m ≠ n → 1 ≤ ∥f m - f n∥) :=
Copy link
Member

Choose a reason for hiding this comment

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

BTW, H can assume that f satisfies ∀ k < n, p (f k) and ∀ k l, k < l → l < n → r (f k) (f l).

src/analysis/normed_space/riesz_lemma.lean Outdated Show resolved Hide resolved
sgouezel and others added 2 commits September 12, 2021 08:46
Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
@urkud
Copy link
Member

urkud commented Sep 15, 2021

Thanks! 🎉
bors merge

@github-actions github-actions bot added ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) and removed awaiting-review The author would like community review of the PR labels Sep 15, 2021
bors bot pushed a commit that referenced this pull request Sep 15, 2021
@bors
Copy link

bors bot commented Sep 15, 2021

Pull request successfully merged into master.

Build succeeded:

1 similar comment
@bors
Copy link

bors bot commented Sep 15, 2021

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(analysis/normed_space/finite_dimension): Riesz theorem on compact unit ball and finite dimension [Merged by Bors] - feat(analysis/normed_space/finite_dimension): Riesz theorem on compact unit ball and finite dimension Sep 15, 2021
@bors bors bot closed this Sep 15, 2021
@bors bors bot deleted the riesz_compact branch September 15, 2021 02:43
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

3 participants