This theory deals with some concrete examples of topologies.
In this section we define and prove the basic properties of the co-cardinal topology on a set \(X\).
The collection of subsets of a set whose complement is strictly bounded by a cardinal is a topology given some assumptions on the cardinal.
definition
\( \text{CoCardinal}(X,T) \equiv \{F\in Pow(X).\ X-F \prec T\}\cup \{0\} \)
For any set and any infinite cardinal we prove that \( \text{CoCardinal}(X,Q) \) forms a topology. The proof is done with an infinite cardinal, but it is obvious that the set Q can be any set equipollent with an infinite cardinal. It is a topology also if the set where the topology is defined is too small or the cardinal too large; in this case, as it is later proved the topology is a discrete topology. And the last case corresponds with \( "Q=1" \) which translates in the indiscrete topology.
lemma CoCar_is_topology:
assumes \( InfCard (Q) \)
shows \( \text{CoCardinal}(X,Q) \text{ is a topology } \)proofWe can use theorems proven in topology0 context for the co-cardinal topology.
theorem topology0_CoCardinal:
assumes \( \text{InfCard}(T) \)
shows \( topology0(\text{CoCardinal}(X,T)) \) using topology0_def, CoCar_is_topology, assmsIt can also be proven that if \( \text{CoCardinal}(X,T) \) is a topology, \( X\neq 0, \text{Card}(T) \) and \( T\neq 0 \); then T is an infinite cardinal, \( X\prec T \) or \( T=1 \). It follows from the fact that the union of two closed sets is closed. Choosing the appropriate cardinals, the cofinite and the cocountable topologies are obtained.
The cofinite topology is a very special topology because it is closely related to the separation axiom \(T_1\). It also appears naturally in algebraic geometry.
definition
\( CoFinite X \equiv \text{CoCardinal}(X,nat) \)
Cocountable topology in fact consists of the empty set and all cocountable subsets of \(X\).
definition
\( CoCountable X \equiv \text{CoCardinal}(X,\text{csucc}(nat)) \)
There are several assertions that can be done to the \( \text{CoCardinal}(X,T) \) topology. In each case, we will not assume sufficient conditions for \( \text{CoCardinal}(X,T) \) to be a topology, but they will be enough to do the calculations in every posible case.
The topology is defined in the set \(X\)
lemma union_cocardinal:
assumes \( T\neq 0 \)
shows \( \bigcup \text{CoCardinal}(X,T) = X \)proofThe closed sets are the small subsets of \(X\) and \(X\) itself.
lemma closed_sets_cocardinal:
assumes \( T\neq 0 \)
shows \( D \text{ is closed in } \text{CoCardinal}(X,T) \longleftrightarrow (D\in Pow(X) \wedge D\prec T) \vee D=X \)proofThe interior of a set is itself if it is open or 0 if it isn't open.
lemma interior_set_cocardinal:
assumes noC: \( T\neq 0 \) and \( A\subseteq X \)
shows \( \text{Interior}(A,\text{CoCardinal}(X,T))= (\text{if }((X-A) \prec T)\text{ then }A\text{ else }0) \)proof\(X\) is a closed set that contains \(A\). This lemma is necessary because we cannot use the lemmas proven in the topology0 context since \(T\neq 0\) is too weak for \( \text{CoCardinal}(X,T) \) to be a topology.
lemma X_closedcov_cocardinal:
assumes \( T\neq 0 \), \( A\subseteq X \)
shows \( X \in Closed \text{Covers}(A,\text{CoCardinal}(X,T)) \) using ClosedCovers_def using union_cocardinal, closed_sets_cocardinal, assmsThe closure of a set is itself if it is closed or \(X\) if it isn't closed.
lemma closure_set_cocardinal:
assumes \( T\neq 0 \), \( A\subseteq X \)
shows \( \text{Closure}(A,\text{CoCardinal}(X,T))=(\text{if }(A \prec T)\text{ then }A\text{ else }X) \)proofThe boundary of a set is empty if \(A\) and \(X-A\) are closed, X if not \(A\) neither \(X-A\) are closed and; if only one is closed, then the closed one is its boundary.
lemma boundary_cocardinal:
assumes \( T\neq 0 \), \( A\subseteq X \)
shows \( \text{Boundary}(A,\text{CoCardinal}(X,T)) = (\text{if }A\prec T\text{ then }(\text{if } (X-A)\prec T\text{ then }0\text{ else }A)\text{ else }(\text{if } (X-A)\prec T\text{ then }X-A\text{ else }X)) \)proofIf the set is too small or the cardinal too large, then the topology is just the discrete topology.
lemma discrete_cocardinal:
assumes \( X\prec T \)
shows \( \text{CoCardinal}(X,T) = Pow(X) \)proofIf the cardinal is taken as \( T=1 \) then the topology is indiscrete.
lemma indiscrete_cocardinal:
shows \( \text{CoCardinal}(X,1) = \{0,X\} \)proofThe topological subspaces of the \( \text{CoCardinal}(X,T) \) topology are also CoCardinal topologies.
lemma subspace_cocardinal:
shows \( \text{CoCardinal}(X,T) \text{ restricted to } Y = \text{CoCardinal}(Y\cap X,T) \)proofIn this section, we consider all the subsets of a set which have empty intersection with a fixed set.
The excluded set topology consists of subsets of \(X\) that are disjoint with a fixed set \(U\).
definition
\( \text{ExcludedSet}(X,U) \equiv \{F\in Pow(X).\ U \cap F=0\}\cup \{X\} \)
For any set; we prove that \( \text{ExcludedSet}(X,Q) \) forms a topology.
theorem excludedset_is_topology:
shows \( \text{ExcludedSet}(X,Q) \text{ is a topology } \)proofWe can use topology0 when discussing excluded set topology.
theorem topology0_excludedset:
shows \( topology0(\text{ExcludedSet}(X,T)) \) using topology0_def, excludedset_is_topologyChoosing a singleton set, it is considered a point in excluded topology.
definition
\( \text{ExcludedPoint}(X,p) \equiv \text{ExcludedSet}(X,\{p\}) \)
Here we discuss what are closed sets, interior, closure and boundary in excluded set topology.
The topology is defined in the set \(X\)
lemma union_excludedset:
shows \( \bigcup \text{ExcludedSet}(X,T) = X \)proofThe closed sets are those which contain the set \( (X \cap T) \) and 0.
lemma closed_sets_excludedset:
shows \( D \text{ is closed in }\text{ExcludedSet}(X,T) \longleftrightarrow (D\in Pow(X) \wedge (X \cap T) \subseteq D) \vee D=0 \)proofThe interior of a set is itself if it is X or the difference with the set T
lemma interior_set_excludedset:
assumes \( A\subseteq X \)
shows \( \text{Interior}(A,\text{ExcludedSet}(X,T)) = (\text{if }A=X\text{ then }X\text{ else }A-T) \)proofThe closure of a set is itself if it is 0 or the union with T.
lemma closure_set_excludedset:
assumes \( A\subseteq X \)
shows \( \text{Closure}(A,\text{ExcludedSet}(X,T))=(\text{if }A=0\text{ then }0\text{ else }A \cup (X\cap T)) \)proofThe boundary of a set is 0 if \(A\) is X or 0, and \( X\cap T \) in other case.
lemma boundary_excludedset:
assumes \( A\subseteq X \)
shows \( \text{Boundary}(A,\text{ExcludedSet}(X,T)) = (\text{if }A=0\vee A=X\text{ then }0\text{ else }X\cap T) \)proofThis section provides some miscellaneous facts about excluded set topologies.
The excluded set topology is equal in the sets T and \( X\cap T \).
lemma smaller_excludedset:
shows \( \text{ExcludedSet}(X,T) = \text{ExcludedSet}(X,(X\cap T)) \)proofIf the set which is excluded is disjoint with X, then the topology is discrete.
lemma empty_excludedset:
assumes \( T\cap X=0 \)
shows \( \text{ExcludedSet}(X,T) = Pow(X) \)proofThe topological subspaces of the ExcludedSet X T topology are also ExcludedSet topologies.
lemma subspace_excludedset:
shows \( \text{ExcludedSet}(X,T) \text{ restricted to } Y = \text{ExcludedSet}(Y \cap X, T) \)proofIn this section we consider the subsets of a set which contain a fixed set. The family defined in this section and the one in the previous section are dual; meaning that the closed set of one are the open sets of the other.
We define the included set topology as the collection of supersets of some fixed subset of the space \(X\).
definition
\( \text{IncludedSet}(X,U) \equiv \{F\in Pow(X).\ U \subseteq F\} \cup \{0\} \)
In the next theorem we prove that IncludedSet X Q forms a topology.
theorem includedset_is_topology:
shows \( \text{IncludedSet}(X,Q) \text{ is a topology } \)proofWe can reference the theorems proven in the topology0 context when discussing the included set topology.
theorem topology0_includedset:
shows \( topology0(\text{IncludedSet}(X,T)) \) using topology0_def, includedset_is_topologyChoosing a singleton set, it is considered a point excluded topology. In the following lemmas and theorems, when neccessary it will be considered that \( T\neq 0 \) and \( T\subseteq X \). These cases will appear in the special cases section.
definition
\( IncludedPoint X p \equiv \text{IncludedSet}(X,\{p\}) \)
This section discusses total set, closed sets, interior, closure and boundary for included set topology.
The topology is defined in the set \(X\).
lemma union_includedset:
assumes \( T\subseteq X \)
shows \( \bigcup \text{IncludedSet}(X,T) = X \)proofThe closed sets are those which are disjoint with T and X.
lemma closed_sets_includedset:
assumes \( T\subseteq X \)
shows \( D \text{ is closed in } \text{IncludedSet}(X,T) \longleftrightarrow (D\in Pow(X) \wedge (D \cap T)=0)\vee D=X \)proofThe interior of a set is itself if it is open or the empty set if it isn't.
lemma interior_set_includedset:
assumes \( A\subseteq X \)
shows \( \text{Interior}(A,\text{IncludedSet}(X,T))= (\text{if }T\subseteq A\text{ then }A\text{ else }0) \)proofThe closure of a set is itself if it is closed or the whole space if it is not.
lemma closure_set_includedset:
assumes \( A\subseteq X \), \( T\subseteq X \)
shows \( \text{Closure}(A,\text{IncludedSet}(X,T)) = (\text{if }T\cap A=0\text{ then }A\text{ else }X) \)proofThe boundary of a set is \( X-A \) if \(A\) contains T completely, is A if \(X-A\) contains T completely and X if T is divided between the two sets. The case where \( T=0 \) is considered as a special case.
lemma boundary_includedset:
assumes \( A\subseteq X \), \( T\subseteq X \), \( T\neq 0 \)
shows \( \text{Boundary}(A,\text{IncludedSet}(X,T))=(\text{if }T\subseteq A\text{ then }X-A\text{ else }(\text{if }T\cap A=0\text{ then }A\text{ else }X)) \)proofIn this section we discuss some corner cases when some parameters in our definitions are empty and provide some facts about subspaces in included set topologies.
The topology is discrete if \( T=0 \)
lemma smaller_includedset:
shows \( \text{IncludedSet}(X,0) = Pow(X) \)proofIf the set which is included is not a subset of X, then the topology is trivial.
lemma empty_includedset:
assumes \( \neg (T\subseteq X) \)
shows \( \text{IncludedSet}(X,T) = \{0\} \)proofThe topological subspaces of the \( \text{IncludedSet}(X,T) \) topology are also IncludedSet topologies. The trivial case does not fit the idea in the demonstration because if \( Y\subseteq X \) then \( \text{IncludedSet}(Y\cap X, Y\cap T) \) is never trivial. There is no need for a separate proof because the only subspace of the trivial topology is itself.
lemma subspace_includedset:
assumes \( T\subseteq X \)
shows \( \text{IncludedSet}(X,T) \text{ restricted to } Y = \text{IncludedSet}(Y\cap X,Y\cap T) \)proofassumes \( A\prec Q \) and \( B\prec Q \) and \( \text{InfCard}(Q) \)
shows \( A \cup B\prec Q \)assumes \( InfCard (Q) \)
shows \( \text{CoCardinal}(X,Q) \text{ is a topology } \)assumes \( T\neq 0 \)
shows \( \bigcup \text{CoCardinal}(X,T) = X \)assumes \( T\neq 0 \)
shows \( D \text{ is closed in } \text{CoCardinal}(X,T) \longleftrightarrow (D\in Pow(X) \wedge D\prec T) \vee D=X \)assumes \( T\neq 0 \), \( A\subseteq X \)
shows \( X \in Closed \text{Covers}(A,\text{CoCardinal}(X,T)) \)assumes \( T\neq 0 \), \( A\subseteq X \)
shows \( \text{Closure}(A,\text{CoCardinal}(X,T))=(\text{if }(A \prec T)\text{ then }A\text{ else }X) \)assumes \( A \subseteq \bigcup T \)
shows \( Closed \text{Covers}(A,T) \neq 0 \)assumes \( A\subseteq X \)
shows \( \text{Closure}(A,\text{ExcludedSet}(X,T))=(\text{if }A=0\text{ then }0\text{ else }A \cup (X\cap T)) \)assumes \( T\subseteq X \)
shows \( \bigcup \text{IncludedSet}(X,T) = X \)assumes \( T\subseteq X \)
shows \( D \text{ is closed in } \text{IncludedSet}(X,T) \longleftrightarrow (D\in Pow(X) \wedge (D \cap T)=0)\vee D=X \)assumes \( A \subseteq \bigcup T \)
shows \( A \text{ is closed in } T \longleftrightarrow cl(A) = A \)assumes \( A\subseteq X \), \( T\subseteq X \)
shows \( \text{Closure}(A,\text{IncludedSet}(X,T)) = (\text{if }T\cap A=0\text{ then }A\text{ else }X) \)