Documentation

Mathlib.Topology.ClopenBox

Clopen subsets in cartesian products #

In general, a clopen subset in a cartesian product of topological spaces cannot be written as a union of "clopen boxes", i.e. products of clopen subsets of the components (see [buzyakovaClopenBox] for counterexamples).

However, when one of the factors is compact, a clopen subset can be written as such a union. Our argument in TopologicalSpace.Clopens.exists_prod_subset follows the one given in [buzyakovaClopenBox].

We deduce that in a product of compact spaces, a clopen subset is a finite union of clopen boxes, and use that to prove that the property of having countably many clopens is preserved by taking cartesian products of compact spaces (this is relevant to the theory of light profinite sets).

References #

theorem TopologicalSpace.Clopens.exists_prod_subset {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] [CompactSpace Y] (W : TopologicalSpace.Clopens (X × Y)) {a : X × Y} (h : a W) :
∃ (U : TopologicalSpace.Clopens X), a.1 U ∃ (V : TopologicalSpace.Clopens Y), a.2 V U ×ˢ V W

Every clopen set in a product of two compact spaces is a union of finitely many clopen boxes.