Zulip Chat Archive

Stream: Is there code for X?

Topic: basis..sum_extend_extends


Adam Topaz (Mar 28 2022 at 17:40):

Do we really not have this lemma?

import linear_algebra.basis

variables {ι K M : Type*} [field K] [add_comm_group M] [module K M]

example (f : ι  M) (hf : linear_independent K f) (i : ι) :
  (basis.sum_extend hf) (sum.inl i) = f i :=
begin
  dsimp [basis.sum_extend],
  simp,
end

Anne Baanen (Mar 29 2022 at 10:22):

Probably not, IIRC most of these basis.extend-form lemmas were defined for their type rather than their evaulation properties.


Last updated: Dec 20 2023 at 11:08 UTC