Commit 2025-02-25 23:58 c28c3dab

View on Github →

chore(LinearAlgebra): split LinearIndependent into Defs, Basic, Lemmas (#22065) I was looking at reducing the imports and non-deffiness of LinearAlgebra.Basis.Defs and one big obstacle is that the basic dependencies in linear algebra already bring in a lot of theory. So I decided to try and split this large file. I ended up with three files:

  • LinearIndependent.Defs contains the definitions and lemmas stating equivalent definitions to linear independence.
  • LinearIndependent.Basic contains results provable without additional imports
  • LinearIndependent.Lemmas contains the rest of the lemmas

Estimated changes

deleted theorem LinearIndepOn.id_image
deleted theorem LinearIndepOn.id_imageₛ
deleted theorem LinearIndepOn.id_union
deleted theorem LinearIndepOn.image
deleted theorem LinearIndepOn.injOn
deleted theorem LinearIndepOn.map_injOn
deleted theorem LinearIndepOn.mono
deleted theorem LinearIndepOn.ne_zero
deleted theorem LinearIndepOn.of_comp
deleted theorem LinearIndepOn.singleton
deleted def LinearIndepOn
deleted theorem LinearIndependent.comp
deleted theorem LinearIndependent.map'
deleted theorem LinearIndependent.map
deleted theorem LinearIndependent.ne_zero
deleted theorem LinearIndependent.of_comp
deleted theorem LinearIndependent.option
deleted theorem LinearIndependent.repr_eq
deleted def LinearIndependent
deleted theorem exists_linearIndependent'
deleted theorem exists_linearIndependent
deleted theorem le_of_span_le_span
deleted theorem linearDepOn_iff'
deleted theorem linearDepOn_iff'ₛ
deleted theorem linearDepOn_iff
deleted theorem linearDepOn_iffₛ
deleted theorem linearIndepOn_empty
deleted theorem linearIndepOn_equiv
deleted theorem linearIndepOn_id_insert
deleted theorem linearIndepOn_id_pair
deleted theorem linearIndepOn_iff
deleted theorem linearIndepOn_iff_image
deleted theorem linearIndepOn_iffₛ
deleted theorem linearIndepOn_insert
deleted theorem linearIndepOn_of_finite
deleted theorem linearIndepOn_range_iff
deleted theorem linearIndepOn_univ
deleted theorem linearIndependent_empty
deleted theorem linearIndependent_equiv'
deleted theorem linearIndependent_equiv
deleted theorem linearIndependent_fin2
deleted theorem linearIndependent_iff''
deleted theorem linearIndependent_iff'
deleted theorem linearIndependent_iff'ₛ
deleted theorem linearIndependent_iff
deleted theorem linearIndependent_iff_ker
deleted theorem linearIndependent_iffₛ
deleted theorem linearIndependent_option'
deleted theorem linearIndependent_option
deleted theorem linearIndependent_span
deleted theorem linearIndependent_sum
deleted theorem mem_span_insert_exchange
deleted theorem not_linearIndependent_iff
deleted theorem span_le_span_iff
added theorem LinearIndepOn.id_image
added theorem LinearIndepOn.id_union
added theorem LinearIndepOn.image
added theorem LinearIndepOn.mono
added theorem LinearIndependent.map'
added theorem LinearIndependent.map
added theorem le_of_span_le_span
added theorem linearIndependent_span
added theorem linearIndependent_sum
added theorem span_le_span_iff
added theorem LinearIndepOn.injOn
added theorem LinearIndepOn.ne_zero
added theorem LinearIndepOn.of_comp
added def LinearIndepOn
added theorem LinearIndependent.comp
added theorem linearDepOn_iff'
added theorem linearDepOn_iff'ₛ
added theorem linearDepOn_iff
added theorem linearDepOn_iffₛ
added theorem linearIndepOn_empty
added theorem linearIndepOn_equiv
added theorem linearIndepOn_iff
added theorem linearIndepOn_iffₛ
added theorem linearIndepOn_univ
added theorem linearIndependent_iff'
added theorem linearIndependent_iff
added theorem linearIndepOn_id_pair
added theorem linearIndepOn_insert
added theorem linearIndependent_fin2