Zulip Chat Archive
Stream: Is there code for X?
Topic: Linear independent equivalent formulations
Martin Dvořák (Apr 05 2024 at 13:00):
How can we prove that these two formulations of linear independence are equivalent?
import Mathlib
example {ι F : Type} [Field F] {S : Set ι} {f : ι → F} :
LinearIndependent F (f · : S → F) ↔
LinearIndependent F (fun x => x : S.image f → F) := by
sorry
Yaël Dillies (Apr 05 2024 at 13:02):
They are not. Consider S := Set.univ
, f := Function.const Bool 0
Yaël Dillies (Apr 05 2024 at 13:05):
The case that's true is given by docs#linearIndependent_image
Martin Dvořák (Apr 05 2024 at 13:34):
The awkward moment when you realize that Set.image
actually produces a set.
Last updated: May 02 2025 at 03:31 UTC