Zulip Chat Archive
Stream: new members
Topic: Subset of an empty set is empty
Yagub Aliyev (Feb 05 2024 at 09:58):
How to show that a subset of an empty set is empty in Lean? This is my incomplete attempt:
https://adam.math.hhu.de/#/g/hhu-adam/robo/world/SetTheory/level/4
theorem Set.subset_empty_iff {A : Type _} (s : Set A) : s ⊆ ∅ ↔ s = ∅ := by
constructor
rw[imp_iff_not_or]
by_cases h : s = ∅
right
exact h
left
by_contra
have h0 : s=∅ := a
Ruben Van de Velde (Feb 05 2024 at 10:22):
Looking at the available lemmas, Set.Subset.antisymm
looks interesting.
Ruben Van de Velde (Feb 05 2024 at 10:25):
Incidentally, this seems to be what the game suggests itself
Last updated: May 02 2025 at 03:31 UTC