Zulip Chat Archive
Stream: mathlib4
Topic: reindexAlgEquiv
Kevin Buzzard (Jul 17 2024 at 11:10):
Right now docs#Matrix.reindexAlgEquiv is
def reindexAlgEquiv (e : m ≃ n) : Matrix m m R ≃ₐ[R] Matrix n n R :=
for R a CommSemiring. But in fact @Edison Xie pointed out that this can be generalised to
def reindexAlgEquiv (e : m ≃ n) : Matrix m m A ≃ₐ[R] Matrix n n A :=
with [Algebra R A] and A not necessarily commutative (and he needs this for his work on Brauer groups). My question is whether reindexAlgEquiv should be redefined, or whether this new isomorphism should be a new declaration.
Matthew Ballard (Jul 17 2024 at 11:14):
Where is reindexAlgEquiv currently used?
Edison Xie (Jul 17 2024 at 12:48):
Matthew Ballard said:
Where is
reindexAlgEquivcurrently used?
LinearAlgebra.Matrix.Basis and LinearAlgebra.Matrix.Transvection iirc
Eric Wieser (Jul 17 2024 at 13:03):
I think it's fine to generalize it; just make R an explicit argument
Last updated: May 02 2025 at 03:31 UTC