Zulip Chat Archive
Stream: mathlib4
Topic: LinearAlgebra.Span !4#2248
Johan Commelin (Feb 14 2023 at 13:41):
def toSpanNonzeroSingleton (x : V) (h : x ≠ 0) : K ≃ₗ[K] K ∙ x := -- error on the type
-- failed to synthesize instance
-- RingHomInvPair (RingHom.id K) ?m.479207
Johan Commelin (Feb 14 2023 at 13:42):
Adding an instance RingHomInvPair (RingHom.id K) (RingHom.id K)
doesn't even help.
Eric Wieser (Feb 14 2023 at 13:43):
What does it want with pp.explicit true
?
Eric Wieser (Feb 14 2023 at 13:43):
This is surely still the typeclass eta bug
Johan Commelin (Feb 14 2023 at 13:44):
failed to synthesize instance
@RingHomInvPair K K (@DivisionSemiring.toSemiring K (@Semifield.toDivisionSemiring K (@Field.toSemifield K inst✝²)))
(@DivisionSemiring.toSemiring K (@Semifield.toDivisionSemiring K (@Field.toSemifield K inst✝²)))
(@RingHom.id K
(@NonAssocRing.toNonAssocSemiring K
(@Ring.toNonAssocRing K (@DivisionRing.toRing K (@Field.toDivisionRing K inst✝²)))))
?m.479207
Johan Commelin (Feb 14 2023 at 13:44):
Aha, I see NonAssocRing
. So maybe the fix that @Pol'tta / Kô Miyahara found will work here as well
Johan Commelin (Feb 14 2023 at 13:47):
Yep, that helps!
Johan Commelin (Feb 14 2023 at 13:48):
file is now error-free
Eric Wieser (Feb 14 2023 at 13:51):
Do you remember the issue number I'm thinking of?
Johan Commelin (Feb 14 2023 at 13:52):
Last updated: Dec 20 2023 at 11:08 UTC