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.
lean4game/server/testgame/TestGame/Levels/SetTheory/L09_Complement.lean

36 lines
675 B
Plaintext

This file contains ambiguous Unicode characters!

This file contains ambiguous Unicode characters that may be confused with others in your current locale. If your use case is intentional and legitimate, you can safely ignore this warning. Use the Escape button to highlight these characters.

import TestGame.Metadata
import Mathlib.Data.Set.Basic
Game "TestGame"
World "SetTheory"
Level 9
Title "Komplement"
Introduction
"
Das Komplement einer Menge wird als `Aᶜ` (`\\^c`) geschrieben. Wichtige Lemmas
sind `not_mem_compl_iff` und `compl_eq_univ_diff`.
"
open Set
#check not_mem_compl_iff
#check compl_eq_univ_diff
Statement
""
(A : Set ) (h : Aᶜ ⊆ A) : A = univ := by
apply Subset.antisymm
simp only [subset_univ]
intros x hx
by_cases h4 : x ∈ Aᶜ
exact mem_of_subset_of_mem h h4
rw [←not_mem_compl_iff]
exact h4
NewTactics constructor intro rw assumption rcases simp tauto trivial
NewLemmas Subset.antisymm_iff empty_subset