Skip to content

Commit

Permalink
feat(analysis/normed_space/real_inner_product): linear independence o…
Browse files Browse the repository at this point in the history
…f orthogonal vectors (#4045)

Add the lemma that an indexed family of nonzero, pairwise orthogonal
vectors is linearly independent.
  • Loading branch information
jsm28 committed Sep 6, 2020
1 parent 1117ae7 commit de03e19
Showing 1 changed file with 18 additions and 0 deletions.
18 changes: 18 additions & 0 deletions src/analysis/normed_space/real_inner_product.lean
Expand Up @@ -351,6 +351,24 @@ begin
linarith
end

/-- A family of vectors is linearly independent if they are nonzero
and orthogonal. -/
lemma linear_independent_of_ne_zero_of_inner_eq_zero {ι : Type*} {v : ι → α}
(hz : ∀ i, v i ≠ 0) (ho : ∀ i j, i ≠ j → inner (v i) (v j) = 0) : linear_independent ℝ v :=
begin
rw linear_independent_iff',
intros s g hg i hi,
have h' : g i * inner (v i) (v i) = inner (∑ j in s, g j • v j) (v i),
{ rw sum_inner,
symmetry,
convert finset.sum_eq_single i _ _,
{ rw inner_smul_left },
{ intros j hj hji,
rw [inner_smul_left, ho j i hji, mul_zero] },
{ exact λ h, false.elim (h hi) } },
simpa [hg, hz] using h'
end

end basic_properties

section norm
Expand Down

0 comments on commit de03e19

Please sign in to comment.