Zulip Chat Archive

Stream: new members

Topic: standard basis


Hans Parshall (Jan 19 2022 at 04:26):

I would like to show that the standard basis is orthonormal, and I get to a reasonable looking statement in terms of function.update:

import analysis.inner_product_space.basic
import analysis.inner_product_space.pi_L2
import analysis.normed_space.pi_Lp

variables {F m : Type*}
  [is_R_or_C F]
  [fintype m]
  [decidable_eq m]
  [inner_product_space F (m  F)]

lemma bm_on : orthonormal F (pi.basis_fun F m) :=
begin
  rw orthonormal,
  split,
  intro i,
  {
    rw pi.basis_fun,
    simp,
    sorry,
  },
  intros i j,
  intro neq,
  {
    rw pi.basis_fun,
    simp,
    sorry,
  },
end

I am having difficulty getting function.update to interact with inner. Any help is appreciated!

Kevin Buzzard (Jan 19 2022 at 04:37):

Doesn't variable [inner_product_space F (m → F)] mean "assume there is a completely arbitrary inner product space structure on m → F about which we know nothing"? If so then your lemma will not be true. I'm not 100% sure of this though, I don't know this part of the library.

Hans Parshall (Jan 19 2022 at 16:30):

This does seem like an issue. How do I specialize?

Heather Macbeth (Jan 19 2022 at 16:34):

You should use docs#euclidean_space !

Hans Parshall (Jan 19 2022 at 17:17):

How do I access the standard basis for euclidean_space ?

Heather Macbeth (Jan 19 2022 at 17:24):

Something like (ite (i = j) (1:𝕜) 0 : euclidean_space 𝕜 m), although I'd be curious to know what your use case is ... do you really need a basis for it?

Hans Parshall (Jan 19 2022 at 17:27):

The current use case is practicing Lean and navigating mathlib; I think that my original reason for wanting this basis is obsolete, but it still feels like an exercise that I should be able to accomplish.

Hans Parshall (Jan 19 2022 at 17:29):

I am still very new to this and appreciate your help!

Yaël Dillies (Jan 19 2022 at 17:40):

Precisely, you can use docs#pi.single

Hans Parshall (Jan 19 2022 at 17:51):

I think this is what pi.basis_fun does. How do I work with this in euclidean space?


Last updated: Dec 20 2023 at 11:08 UTC