Kuratowski's closure-complement theorem is sharp #
Kuratowski's closure-complement theorem 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.
This file gives an example of a so-called "14-set" in ℝ, from which exactly 14 distinct sets can be obtained.
Our strategy is to show there is no duplication within the fourteen sets obtained from this set
s
: the fourteen sets can be decomposed into six closed sets, six open sets that are the
complements of the closed sets, and s
and sᶜ
which are neither closed nor open.
This reduces 14*13/2 = 91
inequalities to check down to 6*5/2 = 15
inequalities.
We'll further show that the 15 inequalities follow from a subset of 6 by algebra.
There are charaterizations and criteria for a set to be a 14-set in the paper "Characterization of Kuratowski 14-Sets" by Eric Langford which we do not formalize.
Main definitions #
Topology.ClosureCompl.fourteenSet
: an explicit example of a 14-set in ℝ.Topology.ClosureCompl.theClosedSix
: the six open sets obtainable from a given set.Topology.ClosureCompl.theOpenSix
: the six open sets obtainable from a given set.Topology.ClosureCompl.TheSixIneq
: six inequalities that suffice to deduce that the six closed sets obtained from a given set contain no duplicates.
Main results #
Topology.ClosureCompl.nodup_theFourteen_fourteenSet
: the application of all 14 operations on the definedfourteenSet
in ℝ gives no duplicates.Topology.ClosureCompl.ncard_isObtainable_fourteenSet
: for the definedfourteenSet
in ℝ, there are exactly 14 distinct sets that can be obtained fromfourteenSet
using the closure and complement operations.
The six closed sets obtained from a given set s
are given by applying
k, kc, kck, kckc, kckck, kckckc
to s
.
Equations
Instances For
The complements of the six closed sets.
Equations
Instances For
theFourteen s
can be splitted into 3 subsets.
Every set in theClosedSix s
is closed (because the last operation is closure).
Every set in theOpenSix s
is open.
Six inequalities that suffice to deduce the six closed sets obtained from a given set contain no duplicates.
Equations
- One or more equations did not get rendered due to their size.
Instances For
theClosedSix
applied to an arbitrary set s
results in no duplicates iff TheSixIneq
is true for s
.
theFourteen s
contains no duplicates if and only if theClosedSix s
has none,
and theClosedSix s
is disjoint from theOpenSix s
.
Let the fourteenSet be s: (0,1) ∪ (1,2) ∪ {3} ∪ ([4,5] ∩ ℚ)
Then the following sets can be obtained via the closure and complement operations:
cs = (-∞,0] ∪ {1} ∪ [2,3) ∪ (3,4) ∪ ([4,5] \ ℚ) ∪ (5,∞)
kcs = (-∞,0] ∪ {1} ∪ [2,∞)
ckcs = (0,1) ∪ (1,2)
kckcs = [0,2]
ckckcs = (-∞,0) ∪ (2,∞)
kckckcs = (-∞,0] ∪ [2,∞)
ckckckcs = (0,2)
ks = [0,2] ∪ {3} ∪ [4,5]
cks = (-∞,0) ∪ (2,3) ∪ (3,4) ∪ (5,∞)
kcks = (-∞,0] ∪ [2,4] ∪ [5,∞)
ckcks = (0,2) ∪ (4,5)
kckcks = [0,2] ∪ [4,5]
ckckcks = (-∞,0) ∪ (2,4) ∪ (5,∞)
We can see that the sets are pairwise distinct, so we have 14 distinct sets.
theClosedSix
applied to the specific fourteenSet
generates no duplicates.
No set from theClosedSix fourteenSet
is empty.
No set from theClosedSix fourteenSet
is the universal set.
The fourteen different operations applied to the fourteenSet
generate no duplicates.
The number of distinct sets obtainable from fourteenSet
is exactly 14.