Zulip Chat Archive
Stream: Is there code for X?
Topic: Quotient of Pi type equivalent to Pi of quotient type
Praneeth Kolichala (Dec 16 2021 at 02:21):
I see there is a pi_setoid
(https://github.com/leanprover-community/mathlib/blob/93047c523782a1cf6d1e96dc55beeab88c63d0ab/src/data/quot.lean#L252) in mathlib, but the natural followup would be something like:
lemma pi_quotient_equiv_quotient_pi
{I : Type} {α : I → Type} [∀ i, setoid (α i)] :
(Π i, @quotient (α i) infer_instance) ≃ @quotient (Π i, (α i)) infer_instance
:= sorry
Does such a thing exist? If not, I'm having trouble writing it; I want a function which descends to the quotient within a pi type, but I don't know how to do that without already having something like this function.
In other words, if you have a function such that depends on each coordinate of the input only up to some equivalence relation , how do you descend to ?
Last updated: Dec 20 2023 at 11:08 UTC