Zulip Chat Archive
Stream: Is there code for X?
Topic: Non-dependent exists
Marcus Rossel (Nov 13 2024 at 15:51):
Does such a theorem exist somewhere?
example : (∃ _ : p, q) ↔ p ∧ q where
mp := fun ⟨hp, hq⟩ => ⟨hp, hq⟩
mpr := fun ⟨hp, hq⟩ => ⟨hp, hq⟩
Kyle Miller (Nov 13 2024 at 15:51):
example : (∃ _ : p, q) ↔ p ∧ q := by
exact? -- Try this: exact exists_prop
Marcus Rossel (Nov 13 2024 at 15:55):
Huh, I thought I tried that. Thanks!
Last updated: May 02 2025 at 03:31 UTC