One of the facts demonstrated in every class on General Topology is that in a \(T_2\) (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 \(y\in K^c\). Since \(X\) is \(T_2\), for every point \(x\in K\) we can find an open set \(U_x\) such that \(y\notin \overline{U_x}\). Obviously \(\{U_x\}_{x\in K}\) 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 \(T_2\) spaces, if \(x\neq y\), then there is an open set \(U\) such that \(x\in U\) and \(y\notin \overline{U}\)" (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 \(\{U_x \}_{x\in K}\) in this proof we have to select one such set among many for every \(x\in K\) and this is where we use the Axiom of Choice. Probably in 99/100 cases when an informal calculus proof states something like \(\forall \varepsilon \exists \delta_\varepsilon \cdots\) 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 \(T_2\) space compact sets are closed.
In this section we show that in a \(T_2\) topological space compact sets are closed.
First we prove a lemma that in a \(T_2\) space two points can be separated by the closure of an open set.
lemma (in topology0) T2_cl_open_sep:
assumes \( T \text{ is }T_2 \) and \( x \in \bigcup T \), \( y \in \bigcup T \), \( x\neq y \)
shows \( \exists U\in T.\ (x\in U \wedge y \notin cl(U)) \)proofAC-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 \( \text{FinPow}(A) \) denotes the set of finite subsets of \(A\) in IsarMathLib.
theorem (in topology0) in_t2_compact_is_cl:
assumes A1: \( T \text{ is }T_2 \) and A2: \( K \text{ is compact in } T \)
shows \( K \text{ is closed in } T \)proofassumes \( A \subseteq \bigcup T \), \( V\in T \) and \( A\cap V = 0 \)
shows \( cl(A) \cap V = 0 \)assumes \( T \text{ is }T_2 \) and \( x \in \bigcup T \), \( y \in \bigcup T \), \( x\neq y \)
shows \( \exists U\in T.\ (x\in U \wedge y \notin cl(U)) \)assumes \( A \subseteq \bigcup T \)
shows \( cl(A) \text{ is closed in } T \) and \( \bigcup T - cl(A) \in T \)assumes \( \forall V\in B.\ K(V)\in C \) and \( N \in \text{FinPow}(B) \)
shows \( \{K(V).\ V\in N\} \in \text{FinPow}(C) \)assumes \( N \in \text{FinPow}(\{D\in Pow(\bigcup T).\ D \text{ is closed in } T\}) \)
shows \( (\bigcup N) \text{ is closed in } T \)assumes \( A \subseteq \bigcup T \)
shows \( A \subseteq cl(A) \)assumes \( \forall x\in V.\ \exists U\in T.\ (x\in U \wedge U\subseteq V) \)
shows \( V\in T \)