The Kuratowski closure-complement theorem #
This file proves Kuratowski's closure-complement theorem, which says that if one repeatedly applies the closure and complement operators to a set in a topological space, at most 14 distinct sets can be obtained.
In another file it will be shown that the maximum can be realized in the real numbers. (A set realizing the maximum is called a 14-set.)
Main definitions #
Topology.ClosureCompl.IsObtainable
is the binary inductive predicate saying that a set can be obtained from another using the closure and complement operations.Topology.ClosureCompl.theFourteen
is an explicit multiset of fourteen sets obtained from a given set using the closure and complement operations.
Main results #
Topology.ClosureCompl.mem_theFourteen_iff_isObtainable
: a sett
is obtainable by froms
if and only if they are in the MultisettheFourteen s
.Topology.ClosureCompl.ncard_isObtainable_le_fourteen
: for an arbitrary sets
, there are at most 14 distinct sets that can be obtained froms
using the closure and complement operations (the Kuratowski closure-complement theorem).
Notation #
k
: the closure of a set.i
: the interior of a set.c
: the complement of a set in docstrings;ᶜ
is used in the code.
References #
- https://en.wikipedia.org/wiki/Kuratowski%27s_closure-complement_problem
- https://web.archive.org/web/20220212062843/http://nzjm.math.auckland.ac.nz/images/6/63/The_Kuratowski_Closure-Complement_Theorem.pdf
IsObtainable s t
means that t
can be obtained from s
by taking closures and complements.
- base {X : Type u_1} [TopologicalSpace X] {s : Set X} : IsObtainable s s
- closure {X : Type u_1} [TopologicalSpace X] {s : Set X} ⦃t : Set X⦄ : IsObtainable s t → IsObtainable s (closure t)
- complement {X : Type u_1} [TopologicalSpace X] {s : Set X} ⦃t : Set X⦄ : IsObtainable s t → IsObtainable s tᶜ
Instances For
Equations
- Topology.ClosureCompl.termK = Lean.ParserDescr.node `Topology.ClosureCompl.termK 1024 (Lean.ParserDescr.symbol "k")
Instances For
Equations
- Topology.ClosureCompl.termI = Lean.ParserDescr.node `Topology.ClosureCompl.termI 1024 (Lean.ParserDescr.symbol "i")
Instances For
The at most fourteen sets that are obtainable from s
are given by applying
id, c, k, ck, kc, ckc, kck, ckck, kckc, ckckc, kckck, ckckck, kckckc, ckckckc
to s
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
theFourteen
has exactly 14 sets (possibly with repetition) in it.
If t
is obtainable from s
by the closure and complement operations,
then it is in the multiset theFourteen s
.
A set t
is obtainable by from s
if and only if they are in the Multiset theFourteen s
.
Kuratowski's closure-complement theorem: the number of obtainable sets via closure and
complement operations from a single set s
is at most 14.