Zulip Chat Archive

Stream: new members

Topic: Show that z is in a1


Shadman Sakib (Aug 19 2021 at 15:23):

How do I prove that z in a vector space is an element of a1a_1 which is in a subspace R V?

Shadman Sakib (Aug 19 2021 at 15:24):

import analysis.complex.circle
import analysis.normed_space.inner_product

noncomputable theory

open complex
variables {V : Type*} [inner_product_space  V]

example {V : Type u_1}
  [inner_product_space  V]
  (a₁ : subspace  V)
  [complete_space a₁]
  (z : V) :
  z  a₁ :=
begin
  admit,
end

Eric Wieser (Aug 19 2021 at 15:30):

What's the t argument doing there?

Shadman Sakib (Aug 19 2021 at 15:32):

Sorry, you are right, we do not need that

Eric Wieser (Aug 19 2021 at 15:34):

What's your maths proof?

Eric Wieser (Aug 19 2021 at 15:35):

Because this similar statement is obviously false:

example {V : Type u_1} [add_comm_monoid V] [module  V]
  (a₁ : subspace  V)
  (z : V) :
  z  a₁ :=
begin
  -- false, pick `V = ℝ`, `a₁ = ⊥`, `z = 37`
end

Shadman Sakib (Aug 19 2021 at 15:40):

Z does not always have to be in a1a_1, but z can be on the line a1a_1; I do not have maths proof because I do not know how to prove this goal.

Kyle Miller (Aug 19 2021 at 15:44):

In math english your example is saying "For every subspace a_1 of a vector space V, and for every z in V, then z is in a_1." This is not in general true, unless we know more about a_1. What's the bigger picture of what you're trying to prove?

Eric Rodriguez (Aug 19 2021 at 15:45):

do you mean ∀ V, ∃ a₁ : subspace ℝ V, z ∈ a₁?

Shadman Sakib (Aug 19 2021 at 15:49):

Yeah @Eric Rodriguez that reflects what I'm trying to say much clearer

Eric Wieser (Aug 19 2021 at 15:50):

That means something very different though. The question is once again "what's your maths proof?".

Shadman Sakib (Aug 19 2021 at 15:53):

Sorry, I will get back to you

Eric Wieser (Aug 19 2021 at 16:05):

but z can be on the line a1a_1

This is your maths proof, right? "choose a1a_1 as the line through z, result is trivial"

Eric Wieser (Aug 19 2021 at 16:06):

Eric Rodriguez said:

do you mean ∀ V, ∃ a₁ : subspace ℝ V, z ∈ a₁?

Missing z, ∀ z : V, ∃ a₁ : subspace ℝ V, z ∈ a₁.

Shadman Sakib (Aug 19 2021 at 18:21):

I presume a1a_1 is a fixed line, since there is a specific a1:subspaceRVa_1 : subspace ℝ V given to us

Eric Wieser (Aug 19 2021 at 18:36):

"given to us" is not what "exists" means in the goal


Last updated: Dec 20 2023 at 11:08 UTC