IsarMathLib

Proofs by humans, for humans, formally verified by Isabelle/ZF proof assistant

theory Topology_ZF_1b imports Topology_ZF_1
begin

One of the facts demonstrated in every class on General Topology is that in a T2 (Hausdorff) topological space compact sets are closed. Formalizing the proof of this fact gave me an interesting insight into the role of the Axiom of Choice (AC) in many informal proofs.

A typical informal proof of this fact goes like this: we want to show that the complement of K is open. To do this, choose an arbitrary point yKc. Since X is T2, for every point xK we can find an open set Ux such that yUx. Obviously {Ux}xK covers K, so select a finite subcollection that covers K, and so on. I had never realized that such reasoning requires the Axiom of Choice. Namely, suppose we have a lemma that states "In T2 spaces, if xy, then there is an open set U such that xU and yU" (like our lemma T2_cl_open_sep below). This only states that the set of such open sets U is not empty. To get the collection {Ux}xK in this proof we have to select one such set among many for every xK and this is where we use the Axiom of Choice. Probably in 99/100 cases when an informal calculus proof states something like εδε the proof uses AC. Most of the time the use of AC in such proofs can be avoided. This is also the case for the fact that in a T2 space compact sets are closed.

Compact sets are closed - no need for AC

In this section we show that in a T2 topological space compact sets are closed.

First we prove a lemma that in a T2 space two points can be separated by the closure of an open set.

lemma (in topology0) T2_cl_open_sep:

assumes T is T2 and xT, yT, xy

shows UT. (xUycl(U))proof

AC-free proof that in a Hausdorff space compact sets are closed. To understand the notation recall that in Isabelle/ZF Pow(A) is the powerset (the set of subsets) of A and FinPow(A) denotes the set of finite subsets of A in IsarMathLib.

theorem (in topology0) in_t2_compact_is_cl:

assumes A1: T is T2 and A2: K is compact in T

shows K is closed in Tproof
end