Skip to content

Commit

Permalink
feat(LinearAlgebra/LinearIndependent): add `linearIndependent_iff_fin…
Browse files Browse the repository at this point in the history
…set_linearIndependent` (#9797)

A family is linearly independent if and only if all of its finite subfamily is linearly independent.
  • Loading branch information
acmepjz committed Jan 19, 2024
1 parent f4c4ca6 commit 4bb560b
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions Mathlib/LinearAlgebra/LinearIndependent.lean
Expand Up @@ -238,6 +238,14 @@ theorem LinearIndependent.comp (h : LinearIndependent R v) (f : ι' → ι) (hf
rw [Finsupp.mapDomain_apply hf]
#align linear_independent.comp LinearIndependent.comp

/-- A family is linearly independent if and only if all of its finite subfamily is
linearly independent. -/
theorem linearIndependent_iff_finset_linearIndependent :
LinearIndependent R v ↔ ∀ (s : Finset ι), LinearIndependent R (v ∘ (Subtype.val : s → ι)) :=
fun H _ ↦ H.comp _ Subtype.val_injective, fun H ↦ linearIndependent_iff'.2 fun s g hg i hi ↦
Fintype.linearIndependent_iff.1 (H s) (g ∘ Subtype.val)
(hg ▸ Finset.sum_attach s fun j ↦ g j • v j) ⟨i, hi⟩⟩

theorem LinearIndependent.coe_range (i : LinearIndependent R v) :
LinearIndependent R ((↑) : range v → M) := by simpa using i.comp _ (rangeSplitting_injective v)
#align linear_independent.coe_range LinearIndependent.coe_range
Expand Down

0 comments on commit 4bb560b

Please sign in to comment.