You cannot select more than 25 topics
Topics must start with a letter or number, can include dashes ('-') and can be up to 35 characters long.
34 lines
706 B
Plaintext
34 lines
706 B
Plaintext
2 years ago
|
import TestGame.Metadata
|
||
|
import TestGame.Levels.SetTheory.L05_Empty
|
||
|
|
||
|
import Mathlib.Data.Set.Basic
|
||
|
|
||
|
set_option tactic.hygienic false
|
||
|
|
||
|
Game "TestGame"
|
||
|
World "SetTheory"
|
||
|
Level 6
|
||
|
|
||
|
Title "Nonempty"
|
||
|
|
||
|
Introduction
|
||
|
"
|
||
|
Das Gegenteil von `A = ∅` ist `A ≠ ∅`, aber in Lean wird der Ausdruck `A.Nonempty` bevorzugt.
|
||
|
Dieser ist dadurch existiert, dass in `A` ein Element existiert: `∃x, x ∈ A`.
|
||
|
|
||
|
Zeige dass die beiden Ausdrücke äquivalent sind:
|
||
|
"
|
||
|
|
||
|
open Set
|
||
|
|
||
|
Statement nonempty_iff_ne_empty
|
||
|
""
|
||
|
{A : Type _} (s : Set A) :
|
||
|
s.Nonempty ↔ s ≠ ∅ := by
|
||
|
rw [Set.Nonempty]
|
||
|
rw [ne_eq, eq_empty_iff_forall_not_mem]
|
||
|
push_neg
|
||
|
rfl
|
||
|
|
||
2 years ago
|
NewTactic constructor intro rw assumption rcases simp tauto trivial
|