Zulip Chat Archive

Stream: general

Topic: regression due to #10199


Yakov Pechersky (Dec 12 2021 at 03:23):

Consider:

import data.matrix.notation
import linear_algebra.matrix

example : (1 : matrix (fin 3) (fin 3) ) = ![![1, 0, 0], ![0, 1, 0], ![0, 0, 1]] :=
begin
  ext i j,
  fin_cases i;
  fin_cases j;
  norm_num [matrix.one_apply],
end

Doesn't work on 7d240ce1, works on daac85454a. Does anyone know what changed precisely? As far as I can tell, lemma only got moved, not deleted.

Eric Wieser (Dec 12 2021 at 09:09):

(#10199)

Yury G. Kudryashov (Dec 12 2021 at 13:12):

Works:

import data.fin.vec_notation

example : ![![1, 0, 0], ![0, 1, 0], ![0, 0, 1]] 2 0 = 0 :=
by simp

Doesn't work:

import data.matrix.notation

example : ![![1, 0, 0], ![0, 1, 0], ![0, 0, 1]] 2 0 = 0 :=
by simp

Yury G. Kudryashov (Dec 12 2021 at 13:13):

With import data.matrix.notation, it applies matrix.cons_val', then gets stuck


Last updated: Dec 20 2023 at 11:08 UTC