Zulip Chat Archive

Stream: Is there code for X?

Topic: Lift composition with quot.mk


Yaël Dillies (Feb 02 2022 at 20:49):

Do we have this anywhere? Is it true?

import data.quot

example {α β : Type*} {s : setoid α} (f : quotient s  β)
  (h :  a b, @setoid.r _ s a b  f (quotient.mk' a) = f (quotient.mk' b)) (x : quotient s) :
  quotient.lift_on' x (f  quotient.mk') h = f x :=
sorry

Yaël Dillies (Feb 02 2022 at 20:58):

It's roughly docs#quotient.lift_on'_mk', but the other way around, somehow.

Yury G. Kudryashov (Feb 02 2022 at 21:03):

Can't find it

Yaël Dillies (Feb 02 2022 at 21:03):

Got it

Yaël Dillies (Feb 02 2022 at 21:03):

example {α β : Type*} {s : setoid α} (f : quotient s  β)
  (h :  a b, @setoid.r _ s a b  f (quotient.mk' a) = f (quotient.mk' b)) (a : quotient s) :
  quotient.lift_on' a (f  quotient.mk') h = f a :=
quotient.induction_on' a $ λ a, rfl

Yaël Dillies (Feb 02 2022 at 21:04):

Is it worth having or does it belong to the too-trivial-to-be-stated realm?

Yury G. Kudryashov (Feb 02 2022 at 21:04):

It isn't more trivial than docs#quotient.lift_on_mk

Yaël Dillies (Feb 02 2022 at 21:05):

Okay, great :smiling_face:

Eric Wieser (Feb 02 2022 at 21:46):

Should lift_on just be marked simp so that it unfolds to lift (same for the primed versions)?


Last updated: Dec 20 2023 at 11:08 UTC