Zulip Chat Archive
Stream: Is there code for X?
Topic: Subset of LI family is LI
Martin Dvořák (Mar 30 2024 at 16:18):
I would like to prove that a subset of linearly-independent family is linearly-independent.
It must already exist in Mathlib, right?
I probably failed to write the statement in an idiomatic way.
import Mathlib
example {ι F : Type} [Field F] {I J : Set ι} (hIJ : I ⊆ J) {f : ι → F}
(hJ : LinearIndependent F (f · : J → F)
) : LinearIndependent F (f · : I → F) :=
sorry
Edward van de Meent (Mar 30 2024 at 16:29):
it looks very similar to docs#LinearIndependent.mono ?
Martin Dvořák (Mar 30 2024 at 16:54):
Thanks!
I will take it from here:
import Mathlib
example {F : Type} [Field F] {D E : Set F} (hIJ : D ⊆ E)
(hJ : LinearIndependent F (Subtype.val : E → F)
) : LinearIndependent F (Subtype.val : D → F) :=
LinearIndependent.mono hIJ hJ
Last updated: May 02 2025 at 03:31 UTC