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/adam/Adam/Levels/SetTheory/L18_SetOf.lean

32 lines
619 B
Plaintext

import Adam.Metadata
import Mathlib.Data.Set.Basic
import Mathlib.Algebra.Parity
import Mathlib
Game "Adam"
World "SetTheory2"
Level 5
Title ""
Introduction
"
Zu der Teilmengen-Schreibweise (`SetOf`) gibt es noch zwei spezielle
Syntax, die abundzu auftreten.
Der erste ist `{ x ∈ S | 0 ≤ x}` ( für z.B `(S : Set )`),
welcher eine Abkürzung für `{ x : | x ∈ S ∧ 0 ≤ x}` ist.
Entsprechend hilft auch hier `setOf_and`.
"
open Set
Statement
"" (S : Set ) :
{ x ∈ (S : Set ) | 0 ≤ x} ⊆ S := by
library_search
NewTactic constructor intro rw assumption rcases simp tauto trivial