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/inner_product_space/pi_L2): norms of basis vectors #19020

Closed
wants to merge 2 commits into from

Conversation

eric-wieser
Copy link
Member

@eric-wieser eric-wieser commented May 15, 2023

This adds ‖euclidean_space.single i (a : 𝕜)‖ = ‖a‖ and other similar results.
They hold more generally for pi_Lp, so they are proven there first.

The statement of linear_isometry_equiv.pi_Lp_congr_left_single has also been corrected to include the missing typecast.


Open in Gitpod

This was originally motivated by #19013, though I think I don't actually need it there after all. I think the results are still worth having though.

@eric-wieser eric-wieser added awaiting-review The author would like community review of the PR t-analysis Analysis (normed *, calculus) labels May 15, 2023
Comment on lines +659 to +679
@[simp]
lemma nnnorm_equiv_symm_single (i : ι) (b : β i) :
‖(pi_Lp.equiv p β).symm (pi.single i b)‖₊ = ‖b‖₊ :=
begin
haveI : nonempty ι := ⟨i⟩,
unfreezingI { induction p using with_top.rec_top_coe },
{ simp_rw [nnnorm_eq_csupr, equiv_symm_apply],
refine csupr_eq_of_forall_le_of_forall_lt_exists_gt (λ j, _) (λ n hn, ⟨i, hn.trans_eq _⟩),
{ obtain rfl | hij := decidable.eq_or_ne i j,
{ rw pi.single_eq_same },
{ rw [pi.single_eq_of_ne' hij, nnnorm_zero],
exact zero_le _ } },
{ rw pi.single_eq_same } },
{ have hp0 : (p : ℝ) ≠ 0,
{ exact_mod_cast (zero_lt_one.trans_le $ fact.out (1 ≤ (p : ℝ≥0∞))).ne' },
rw [nnnorm_eq_sum ennreal.coe_ne_top, ennreal.coe_to_real, fintype.sum_eq_single i,
equiv_symm_apply, pi.single_eq_same, ←nnreal.rpow_mul, one_div, mul_inv_cancel hp0,
nnreal.rpow_one],
intros j hij,
rw [equiv_symm_apply, pi.single_eq_of_ne hij, nnnorm_zero, nnreal.zero_rpow hp0] },
end
Copy link
Member Author

@eric-wieser eric-wieser May 15, 2023

Choose a reason for hiding this comment

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

This one was an annoying case bash, but maybe that's unavoidable since both the norm and pi.single are defined by cases.

Co-authored-by: sgouezel <sebastien.gouezel@univ-rennes1.fr>
@sgouezel
Copy link
Collaborator

bors d+

@bors
Copy link

bors bot commented May 17, 2023

✌️ eric-wieser 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 17, 2023
@eric-wieser
Copy link
Member Author

bors merge

@github-actions github-actions bot added the ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) label May 17, 2023
bors bot pushed a commit that referenced this pull request May 17, 2023
)

This adds `‖euclidean_space.single i (a : 𝕜)‖ = ‖a‖` and other similar results.
They hold more generally for `pi_Lp`, so they are proven there first.

The statement of `linear_isometry_equiv.pi_Lp_congr_left_single` has also been corrected to include the missing typecast.
@bors
Copy link

bors bot commented May 17, 2023

Pull request successfully merged into master.

Build succeeded!

The publicly hosted instance of bors-ng is deprecated and will go away soon.

If you want to self-host your own instance, instructions are here.
For more help, visit the forum.

If you want to switch to GitHub's built-in merge queue, visit their help page.

@bors bors bot changed the title feat(analysis/inner_product_space/pi_L2): norms of basis vectors [Merged by Bors] - feat(analysis/inner_product_space/pi_L2): norms of basis vectors May 17, 2023
@bors bors bot closed this May 17, 2023
@bors bors bot deleted the eric-wieser/pi_L2-orthogonal branch May 17, 2023 14:37
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. ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) t-analysis Analysis (normed *, calculus)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

2 participants