Zulip Chat Archive
Stream: Is there code for X?
Topic: heq_comm
Violeta Hernández (Sep 24 2024 at 15:11):
Are we really missing this?
theorem heq_comm.{u} {α β : Sort u} (a : α) (b : β) : HEq a b ↔ HEq b a := by
constructor <;> rintro ⟨⟩ <;> rfl
Adam Topaz (Sep 24 2024 at 15:15):
do you really need an iff
version, or can you get by with docs#HEq.symm ?
Violeta Hernández (Sep 24 2024 at 15:20):
Actually, symm
does work for my purposes
Kyle Miller (Sep 24 2024 at 15:34):
Maybe we'll have it soon: lean4#5456
Violeta Hernández (Sep 24 2024 at 15:34):
Thanks!
Last updated: May 02 2025 at 03:31 UTC