Zulip Chat Archive

Stream: Is there code for X?

Topic: iUnion is compatible with product of types


Michael Rothgang (Oct 05 2023 at 16:19):

lemma iUnion_product {X Y Z : Type*} (f : X × Y  Set Z) :
   (x : X) (y : Y), (f x, y⟩) =  t : X × Y, (f t) := by sorry

I have a proof locally, but also the nagging feeling this should exist somewhere...

None of exact?, apply?, rw? and aesop find this; this isn't listed on docs#Data.Set.Lattice either (where #find_home says it belongs).

Anatole Dedecker (Oct 05 2023 at 16:30):

docs#iSup_prod but I don’t think we have the set spelling

Michael Rothgang (Oct 05 2023 at 16:35):

Thanks - so I'll send a PR then.

Michael Rothgang (Oct 05 2023 at 16:55):

#7528


Last updated: Dec 20 2023 at 11:08 UTC