Zulip Chat Archive

Stream: Is there code for X?

Topic: simp made no progress in finrank of matrix


Edison Xie (Mar 20 2025 at 01:23):

I have simp made no progress in proving Module.finrank F (Matrix (Fin n) (Fin n) F) = n ^ 2 is this suppose to happen?

Edison Xie (Mar 20 2025 at 01:25):

aesop also failed and the proof is rw[pow_two, Module.finrank_matrix] and then simp I thought this should be an easy simp lemma?

Kim Morrison (Mar 20 2025 at 01:27):

Please post a #mwe.

Edison Xie (Mar 20 2025 at 01:28):

import Mathlib

example (F : Type*) [Field F]: Module.finrank F (Matrix (Fin n) (Fin n) F) = n^2 := by
  simp

Edison Xie (Mar 20 2025 at 01:28):

this would give you the error

Bhavik Mehta (Mar 20 2025 at 02:35):

Edison Xie said:

is this suppose to happen?

This looks expected, both of the lemmas you cite for the rw proof are not marked simp, so I wouldn't expect simp to make progress here. I can see an argument for Module.finrank_matrix being a simp lemma though...

Bhavik Mehta (Mar 20 2025 at 02:38):

Actually, the rank version of this lemma is simp, so it probably makes sense for the finrank one to be too


Last updated: May 02 2025 at 03:31 UTC