Zulip Chat Archive
Stream: general
Topic: quot.mk vs quotient.mk
Patrick Massot (Dec 17 2018 at 18:05):
Do we already have lemma quot_mk_quotient_mk {α :Type*} [setoid α] (a : α) : quot.mk setoid.r a = ⟦a⟧ := rfl
? I need this because rintro
typically produces the left-hand side.
Last updated: Dec 20 2023 at 11:08 UTC