Zulip Chat Archive
Stream: general
Topic: Quotient.eq
Violeta Hernández (Nov 02 2024 at 01:06):
I'm trying to update my Rubik's cube project to Lean v.4.13 and I'm running into an issue with Quotient.eq
. Specifically, the rewrite rw [← Quotient.eq]
at x ≈ y
no longer yields ⟦x⟧ = ⟦y⟧
.
Violeta Hernández (Nov 02 2024 at 01:06):
I imagine this is due to one of @Yuyang Zhao's recent refactors, but I'm not quite sure what the intended fix is. Am I just supposed to not use ≈ notation for quotients?
Violeta Hernández (Nov 02 2024 at 01:08):
Or is the idea that every quotient type declares its own Quotient.eq
lemma using the preferred form of the setoid relation?
Violeta Hernández (Nov 02 2024 at 01:43):
For the moment I fixed my code by simply making .eq
lemmas for the quotients I was working with
Yuyang Zhao (Nov 02 2024 at 05:59):
This is #17594. Currently you can use docs#Quotient.eq_iff_equiv.
Last updated: May 02 2025 at 03:31 UTC