Documentation

Archive.Kuratowski

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 #

Main results #

Notation #

References #

inductive Topology.ClosureCompl.IsObtainable {X : Type u_1} [TopologicalSpace X] (s : Set X) :
Set XProp

IsObtainable s t means that t can be obtained from s by taking closures and complements.

Instances For

    The function kckc is idempotent: kckckckc s = kckc s for any set s. This is because ckc = i and ki is idempotent.

    Cancelling the first applied complement we obtain kckckck s = kck s for any set s.

    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.