This theory defines uniform spaces and proves their basic properties.
Just like a topological space constitutes the minimal setting in which one can speak of continuous functions, the notion of uniform spaces (commonly attributed to André Weil) captures the minimal setting in which one can speak of uniformly continuous functions. In some sense this is a generalization of the notion of metric (or metrizable) spaces and topological groups.
There are several definitions of uniform spaces. The fact that these definitions are equivalent is far from obvious (some people call such phenomenon cryptomorphism). We will use the definition of the uniform structure (or ''uniformity'') based on entourages. This was the original definition by Weil and it seems to be the most commonly used. A uniformity consists of entourages that are binary relations between points of space \(X\) that satisfy a certain collection of conditions, specified below.
definition
\( \Phi \text{ is a uniformity on } X \equiv (\Phi \text{ is a filter on } (X\times X))\) \( \wedge (\forall U\in \Phi .\ id(X) \subseteq U \wedge (\exists V\in \Phi .\ V\circ V \subseteq U) \wedge converse(U) \in \Phi ) \)
Since the whole \(X\times X\) is in a uniformity, a uniformity is never empty.
lemma uniformity_non_empty:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \Phi \neq \emptyset \) using assms unfolding IsUniformity_def, IsFilter_defIf \(\Phi\) is a uniformity on \(X\), then the every element \(V\) of \(\Phi\) is a certain relation on \(X\) (a subset of \(X\times X\)) and is called an ''entourage''. For an \(x\in X\) we call \(V\{ x\}\) a neighborhood of \(x\). The first useful fact we will show is that neighborhoods are non-empty.
lemma neigh_not_empty:
assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \) and \( x\in X \)
shows \( W\{x\} \neq \emptyset \) and \( x \in W\{x\} \)proofThe filter part of the definition of uniformity for easier reference:
lemma unif_filter:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \Phi \text{ is a filter on } (X\times X) \) using assms unfolding IsUniformity_defThe second part of the definition of uniformity for easy reference:
lemma entourage_props:
assumes \( \Phi \text{ is a uniformity on } X \) and \( A\in \Phi \)
shows \( A \subseteq X\times X \), \( id(X) \subseteq A \), \( \exists V\in \Phi .\ V\circ V \subseteq A \), \( converse(A) \in \Phi \)proofThe definition of uniformity states (among other things) that for every member \(U\) of uniformity \(\Phi\) there is another one, say \(V\) such that \(V\circ V\subseteq U\). Sometimes such \(V\) is said to be half the size of \(U\). The next lemma states that \(V\) can be taken to be symmetric.
lemma half_size_symm:
assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \)
shows \( \exists V\in \Phi .\ V\circ V \subseteq W \wedge V=converse(V) \)proofInside every member \(W\) of the uniformity \(\Phi\) we can find one that is symmetric and smaller than a third of size \(W\). Compare with the Metamath's theorem with the same name.
lemma ustex3sym:
assumes \( \Phi \text{ is a uniformity on } X \), \( A\in \Phi \)
shows \( \exists B\in \Phi .\ B\circ (B\circ B) \subseteq A \wedge B=converse(B) \)proofIf \(\Phi\) is a uniformity on \(X\) then every element of \(\Phi\) is a subset of \(X\times X\) whose domain is \(X\).
lemma uni_domain:
assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \)
shows \( W \subseteq X\times X \) and \( domain(W) = X \)proofIf \(\Phi\) is a uniformity on \(X\) and \(W\in \Phi\) the for every \(x\in X\) the image of the singleton \(\{ x\}\) by \(W\) is contained in \(X\). Compare the Metamath's theorem with the same name.
lemma ustimasn:
assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \) and \( x\in X \)
shows \( W\{x\} \subseteq X \) using assms, uni_domain(1)Uniformity \( \Phi \) defines a natural topology on its space \(X\) via the neighborhood system that assigns the collection \(\{V(\{x\}):V\in \Phi\}\) to every point \(x\in X\). In the next lemma we show that if we define a function this way the values of that function are what they should be. This is only a technical fact which is useful to shorten the remaining proofs, usually treated as obvious in standard mathematics.
lemma neigh_filt_fun:
assumes \( \Phi \text{ is a uniformity on } X \)
defines \( \mathcal{M} \equiv \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} \)
shows \( \mathcal{M} :X\rightarrow Pow(Pow(X)) \) and \( \forall x\in X.\ \mathcal{M} (x) = \{V\{x\}.\ V\in \Phi \} \)proofIn the next lemma we show that the collection defined in lemma neigh_filt_fun is a filter on \(X\). The proof is kind of long, but it just checks that all filter conditions hold.
lemma filter_from_uniformity:
assumes \( \Phi \text{ is a uniformity on } X \) and \( x\in X \)
defines \( \mathcal{M} \equiv \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} \)
shows \( \mathcal{M} (x) \text{ is a filter on } X \)proofA rephrasing of filter_from_uniformity: if \(\Phi\) is a uniformity on \(X\), then \(\{V(\{ x\}) | V\in \Phi\}\) is a filter on \(X\) for every \(x\in X\).
lemma unif_filter_at_point:
assumes \( \Phi \text{ is a uniformity on } X \) and \( x\in X \)
shows \( \{V\{x\}.\ V\in \Phi \} \text{ is a filter on } X \) using assms, filter_from_uniformity, ZF_fun_from_tot_val1A frequently used property of filters is that they are "upward closed" i.e. supersets of a filter element are also in the filter. The next lemma makes this explicit for easy reference as applied to the natural filter created from a uniformity.
corollary unif_filter_up_closed:
assumes \( \Phi \text{ is a uniformity on } X \), \( x\in X \), \( U \in \{V\{x\}.\ V\in \Phi \} \), \( W\subseteq X \), \( U\subseteq W \)
shows \( W \in \{V\{x\}.\ V\in \Phi \} \) using assms, filter_from_uniformity, ZF_fun_from_tot_val1 unfolding IsFilter_defThe function defined in the premises of lemma neigh_filt_fun (or filter_from_uniformity) is a neighborhood system. The proof uses the existence of the "half-the-size" neighborhood condition (\( \exists V\in \Phi .\ V\circ V \subseteq U \)) of the uniformity definition, but not the \( converse(U) \in \Phi \) part.
theorem neigh_from_uniformity:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} \text{ is a neighborhood system on } X \)proofWhen we have a uniformity \(\Phi\) on \(X\) we can define a topology on \(X\) in a (relatively) natural way. We will call that topology the \( \text{UniformTopology}(\Phi ) \). We could probably reformulate the definition to skip the \(X\) parameter because if \(\Phi\) is a uniformity on \(X\) then \(X\) can be recovered from (is determined by) \(\Phi\).
definition
\( \text{UniformTopology}(\Phi ,X) \equiv \{U\in Pow(X).\ \forall x\in U.\ U\in \{V\{x\}.\ V\in \Phi \}\} \)
An identity showing how the definition of uniform topology is constructed. Here, the \(M = \{\langle t,\{ V\{ t\} : V\in \Phi\}\rangle : t\in X\}\) is the neighborhood system (a function on \(X\)) created from uniformity \(\Phi\). Then for each \(x\in X\), \(M(x) = \{ V\{ t\} : V\in \Phi\}\) is the set of neighborhoods of \(x\).
lemma uniftop_def_alt:
shows \( \text{UniformTopology}(\Phi ,X) = \{U \in Pow(X).\ \forall x\in U.\ U \in \{\langle t,\{V\{t\}.\ V\in \Phi \}\rangle .\ t\in X\}(x)\} \)proofThe collection of sets constructed in the UniformTopology definition is indeed a topology on \(X\).
theorem uniform_top_is_top:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \text{UniformTopology}(\Phi ,X) \text{ is a topology } \) and \( \bigcup \text{UniformTopology}(\Phi ,X) = X \) using assms, neigh_from_uniformity, uniftop_def_alt, topology_from_neighsIf we have a uniformity \(\Phi\) we can create a neighborhood system from it in two ways. We can create a a neighborhood system directly from \(\Phi\) using the formula \(X \ni x \mapsto \{V\{x\} | x\in X\}\) (see theorem neigh_from_uniformity). Alternatively we can construct a topology from \(\Phi\) as in theorem uniform_top_is_top and then create a neighborhood system from this topology as in theorem neigh_from_topology. The next theorem states that these two ways give the same result.
theorem neigh_unif_same:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} = \text{ neighborhood system of } \text{UniformTopology}(\Phi ,X) \) using assms, neigh_from_uniformity, nei_top_nei_round_trip, uniftop_def_altAnother form of the definition of topology generated from a uniformity.
lemma uniftop_def_alt1:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \text{UniformTopology}(\Phi ,X) = \{U\in Pow(X).\ \forall x\in U.\ \exists W\in \Phi .\ W\{x\} \subseteq U\} \)proofImages of singletons by entourages are neighborhoods of those singletons.
lemma image_singleton_ent_nei:
assumes \( \Phi \text{ is a uniformity on } X \), \( V\in \Phi \), \( x\in X \)
defines \( \mathcal{M} \equiv \text{ neighborhood system of } \text{UniformTopology}(\Phi ,X) \)
shows \( V\{x\} \in \mathcal{M} (x) \)proofThe set neighborhoods of a singleton \(\{ x\}\) where \(x\in X\) consist of images of the singleton by the entourages \(W\in \Phi\). See also the Metamath's theorem with the same name.
lemma utopsnneip:
assumes \( \Phi \text{ is a uniformity on } X \), \( x\in X \)
defines \( \mathcal{S} \equiv \text{ set neighborhood system of } \text{UniformTopology}(\Phi ,X) \)
shows \( \mathcal{S} \{x\} = \{W\{x\}.\ W\in \Phi \} \)proofImages of singletons by entourages are set neighborhoods of those singletons. See also the Metamath theorem with the same name.
corollary utopsnnei:
assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \), \( x\in X \)
defines \( \mathcal{S} \equiv \text{ set neighborhood system of } \text{UniformTopology}(\Phi ,X) \)
shows \( W\{x\} \in \mathcal{S} \{x\} \) using assms, utopsnneipIf \(\Phi\) is a uniformity on \(X\) that generates a topology \(T\), \(R\) is any relation on \(X\) (i.e. \(R\subseteq X\times X\)), \(W\) is a symmetric entourage (i.e. \(W\in \Phi\), and \(W\) is symmetric (i.e. equal to its converse)), then the closure of \(R\) in the product topology is contained the the composition \(V\circ (M \circ V)\). Metamath has a similar theorem with the same name.
lemma utop3cls:
assumes \( \Phi \text{ is a uniformity on } X \), \( R\subseteq X\times X \), \( W\in \Phi \), \( W=converse(W) \)
defines \( J \equiv \text{UniformTopology}(\Phi ,X) \)
shows \( \text{Closure}(R,J\times _tJ) \subseteq W\circ (R\circ W) \)proofUniform spaces are regular (\(T_3\)).
theorem utopreg:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \text{UniformTopology}(\Phi ,X) \text{ is regular } \)proofA base or a fundamental system of entourages of a uniformity \(\Phi\) is a subset of \(\Phi\) that is sufficient to uniquely determine it. This is analogous to the notion of a base of a topology (see Topology_ZF_1 or a base of a filter (see Topology_ZF_4).
A base of a uniformity \(\Phi\) is any subset \(\mathfrak{B}\subseteq \Phi\) such that every entourage in \(\Phi\) contains (at least) one from \(\mathfrak{B}\). The phrase is a base for is already defined to mean a base for a topology, so we use the phrase is a uniform base of here.
definition
\( \mathfrak{B} \text{ is a uniform base of } \Phi \equiv \mathfrak{B} \subseteq \Phi \wedge (\forall U\in \Phi .\ \exists B\in \mathfrak{B} .\ B\subseteq U) \)
Symmetric entourages form a base of the uniformity.
lemma symm_are_base:
assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \{V\in \Phi .\ V = converse(V)\} \text{ is a uniform base of } \Phi \)proofGiven a base of a uniformity we can recover the uniformity taking the supersets. The Supersets constructor is defined in ZF1.
lemma uniformity_from_base:
assumes \( \Phi \text{ is a uniformity on } X \), \( \mathfrak{B} \text{ is a uniform base of } \Phi \)
shows \( \Phi = \text{Supersets}(X\times X,\mathfrak{B} ) \)proofAnalogous to the predicate "satisfies base condition" (defined in Topology_ZF_1) and "is a base filter" (defined in Topology_ZF_4) we can specify conditions for a collection \(\mathfrak{B}\) of subsets of \(X\times X\) to be a base of some uniformity on \(X\). Namely, the following conditions are necessary and sufficient:
1. Intersection of two sets of \(\mathfrak{B}\) contains a set of \(\mathfrak{B}\).
2. Every set of \(\mathfrak{B}\) contains the diagonal of \(X\times X\).
3. For each set \(B_1\in \mathfrak{B}\) we can find a set \(B_2\in \mathfrak{B}\) such that \(B_2\subseteq B_1^{-1}\).
4. For each set \(B_1\in \mathfrak{B}\) we can find a set \(B_2\in \mathfrak{B}\) such that \(B_2\circ B_2 \subseteq B_1\).
The conditions are taken from N. Bourbaki "Elements of Mathematics, General Topology", Chapter II.1., except for the last two that are missing there.
definition
\( \mathfrak{B} \text{ is a uniform base on } X \equiv \) \( (\forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2) \wedge (\forall B\in \mathfrak{B} .\ id(X)\subseteq B) \wedge \) \( (\forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1)) \wedge (\forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1) \wedge \) \( \mathfrak{B} \subseteq Pow(X\times X) \wedge \mathfrak{B} \neq \emptyset \)
The next lemma splits the definition of IsUniformityBaseOn into four conditions to enable more precise references in proofs.
lemma uniformity_base_props:
assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \) using assms unfolding IsUniformityBaseOn_defIf supersets of some collection of subsets of \(X\times X\) form a uniformity, then this collection satisfies the conditions in the definition of IsUniformityBaseOn.
theorem base_is_uniform_base:
assumes \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \text{Supersets}(X\times X,\mathfrak{B} ) \text{ is a uniformity on } X \)
shows \( \mathfrak{B} \text{ is a uniform base on } X \)proofif a nonempty collection of subsets of \(X\times X\) satisfies conditions in the definition of IsUniformityBaseOn then the supersets of that collection form a uniformity on \(X\).
theorem uniformity_base_is_base:
assumes \( X\neq \emptyset \) and \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \text{Supersets}(X\times X,\mathfrak{B} ) \text{ is a uniformity on } X \)proofThe assumption that \(X\) is not empty in uniformity_base_is_base above is neccessary as the assertion is false if \(X\) is empty.
lemma uniform_space_empty:
assumes \( \mathfrak{B} \text{ is a uniform base on } \emptyset \)
shows \( \neg ( \text{Supersets}(\emptyset \times \emptyset ,\mathfrak{B} ) \text{ is a uniformity on } \emptyset ) \)proofassumes \( \Phi \text{ is a uniformity on } X \)
shows \( \Phi \text{ is a filter on } (X\times X) \)assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \)
shows \( \exists V\in \Phi .\ V\circ V \subseteq W \wedge V=converse(V) \)assumes \( \Phi \text{ is a uniformity on } X \) and \( A\in \Phi \)
shows \( A \subseteq X\times X \), \( id(X) \subseteq A \), \( \exists V\in \Phi .\ V\circ V \subseteq A \), \( converse(A) \in \Phi \)assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \)
shows \( W \subseteq X\times X \) and \( domain(W) = X \)assumes \( \forall x\in X.\ b(x) \in Y \)
shows \( \{\langle x,b(x)\rangle .\ x\in X\} : X\rightarrow Y \)assumes \( f:X\rightarrow Y \), \( x\in X \) and \( f = \{\langle x,b(x)\rangle .\ x\in X\} \)
shows \( f(x) = b(x) \) and \( b(x)\in Y \)assumes \( \Phi \text{ is a uniformity on } X \)
defines \( \mathcal{M} \equiv \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} \)
shows \( \mathcal{M} :X\rightarrow Pow(Pow(X)) \) and \( \forall x\in X.\ \mathcal{M} (x) = \{V\{x\}.\ V\in \Phi \} \)assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \) and \( x\in X \)
shows \( W\{x\} \neq \emptyset \) and \( x \in W\{x\} \)assumes \( x \in U\{x\} \) and \( U\{x\} \subseteq C \)
shows \( (U \cup C\times C)\{x\} = C \)assumes \( \Phi \text{ is a uniformity on } X \) and \( x\in X \)
defines \( \mathcal{M} \equiv \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} \)
shows \( \mathcal{M} (x) \text{ is a filter on } X \)assumes \( x\in X \)
shows \( \{\langle x,b(x)\rangle .\ x\in X\}(x)=b(x) \)assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} \text{ is a neighborhood system on } X \)assumes \( \mathcal{M} \text{ is a neighborhood system on } X \)
defines \( T \equiv \{U\in Pow(X).\ \forall x\in U.\ U \in \mathcal{M} (x)\} \)
shows \( T \text{ is a topology } \) and \( \bigcup T = X \)assumes \( \mathcal{M} \text{ is a neighborhood system on } X \)
defines \( T \equiv \{U\in Pow(X).\ \forall x\in U.\ U \in \mathcal{M} (x)\} \)
shows \( (\text{ neighborhood system of } T) = \mathcal{M} \)assumes \( \Phi \text{ is a uniformity on } X \) and \( x\in X \)
shows \( \{V\{x\}.\ V\in \Phi \} \text{ is a filter on } X \)assumes \( \mathfrak{F} \text{ is a filter on } X \)
shows \( 0\notin \mathfrak{F} \), \( X\in \mathfrak{F} \), \( \mathfrak{F} \subseteq Pow(X) \), \( \forall A\in \mathfrak{F} .\ \forall B\in \mathfrak{F} .\ A\cap B\in \mathfrak{F} \) and \( \forall B\in \mathfrak{F} .\ \forall C\in Pow(X).\ B\subseteq C \longrightarrow C\in \mathfrak{F} \)assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \{\langle x,\{V\{x\}.\ V\in \Phi \}\rangle .\ x\in X\} = \text{ neighborhood system of } \text{UniformTopology}(\Phi ,X) \)assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \text{UniformTopology}(\Phi ,X) \text{ is a topology } \) and \( \bigcup \text{UniformTopology}(\Phi ,X) = X \)assumes \( x\in \bigcup T \)
shows \( (\text{ neighborhood system of } T)(x) = (\text{ set neighborhood system of } T)\{x\} \)assumes \( \Phi \text{ is a uniformity on } X \), \( x\in X \)
defines \( \mathcal{S} \equiv \text{ set neighborhood system of } \text{UniformTopology}(\Phi ,X) \)
shows \( \mathcal{S} \{x\} = \{W\{x\}.\ W\in \Phi \} \)assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \text{UniformTopology}(\Phi ,X) \text{ is a topology } \) and \( \bigcup \text{UniformTopology}(\Phi ,X) = X \)assumes \( T \text{ is a topology } \), \( S \text{ is a topology } \)
shows \( (T\times _tS) \text{ is a topology } \), \( \text{ProductCollection}(T,S) \text{ is a base for } (T\times _tS) \), \( \bigcup (T\times _tS) = \bigcup T \times \bigcup S \)assumes \( A \subseteq \bigcup T \)
shows \( cl(A) \subseteq \bigcup T \), \( cl(\bigcup T - A) = \bigcup T - int(A) \)assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \), \( x\in X \)
defines \( \mathcal{S} \equiv \text{ set neighborhood system of } \text{UniformTopology}(\Phi ,X) \)
shows \( W\{x\} \in \mathcal{S} \{x\} \)assumes \( T \text{ is a topology } \), \( S \text{ is a topology } \) and \( A \in (\text{ set neighborhood system of } T)(C) \) and \( B \in (\text{ set neighborhood system of } S)(D) \)
shows \( A\times B \in (\text{ set neighborhood system of } (T\times _tS))(C\times D) \)assumes \( z = \langle x,y\rangle \)
shows \( \{x\}\times \{y\} = \{z\} \)assumes \( T \text{ is a topology } \), \( A\subseteq \bigcup T \), \( x \in \text{Closure}(A,T) \) and \( N \in (\text{ set neighborhood system of } T)\{x\} \)
shows \( N\cap A \neq 0 \)assumes \( W=converse(W) \) and \( (W\{x\})\times (W\{y\}) \cap R \neq \emptyset \)
shows \( \langle x,y\rangle \in (W\circ (R\circ W)) \)assumes \( V\in T \), \( x\in V \)
shows \( V \in (\text{ set neighborhood system of } T)\{x\} \)assumes \( \Phi \text{ is a uniformity on } X \), \( A\in \Phi \)
shows \( \exists B\in \Phi .\ B\circ (B\circ B) \subseteq A \wedge B=converse(B) \)assumes \( \Phi \text{ is a uniformity on } X \), \( W\in \Phi \) and \( x\in X \)
shows \( W\{x\} \subseteq X \)assumes \( N \in (\text{ set neighborhood system of } T)(A) \)
shows \( \exists U\in T.\ (A\subseteq U \wedge U\subseteq N) \)assumes \( \Phi \text{ is a uniformity on } X \) and \( A\in \Phi \)
shows \( A \subseteq X\times X \), \( id(X) \subseteq A \), \( \exists V\in \Phi .\ V\circ V \subseteq A \), \( converse(A) \in \Phi \)assumes \( B \subseteq \bigcup T \) and \( A\subseteq B \)
shows \( cl(A) \subseteq cl(B) \)assumes \( T \text{ is a topology } \), \( S \text{ is a topology } \), \( R \subseteq (\bigcup T)\times (\bigcup S) \), \( x\in \bigcup T \)
shows \( \text{Closure}(R\{x\},S) \subseteq \text{Closure}(R,T\times _tS)\{x\} \)assumes \( \Phi \text{ is a uniformity on } X \), \( R\subseteq X\times X \), \( W\in \Phi \), \( W=converse(W) \)
defines \( J \equiv \text{UniformTopology}(\Phi ,X) \)
shows \( \text{Closure}(R,J\times _tJ) \subseteq W\circ (R\circ W) \)assumes \( T \text{ is a topology } \)
shows \( T \text{ is regular } \longleftrightarrow (\forall W\in T.\ \forall x\in W.\ \exists V\in T.\ x\in V \wedge \text{Closure}(V,T)\subseteq W) \)assumes \( r \subseteq X\times X \), \( id(X) \subseteq r \)
shows \( r \subseteq r\circ r \)assumes \( \Phi \text{ is a uniformity on } X \)
shows \( \Phi \neq \emptyset \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)assumes \( A\subseteq X \), \( A\in \mathcal{A} \)
shows \( A \in \text{Supersets}(X,\mathcal{A} ) \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)assumes \( \mathfrak{B} \text{ is a uniform base on } X \)
shows \( \forall B_1\in \mathfrak{B} .\ \forall B_2\in \mathfrak{B} .\ \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \), \( \forall B\in \mathfrak{B} .\ id(X)\subseteq B \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \), \( \forall B_1\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \), \( \mathfrak{B} \subseteq Pow(X\times X) \) and \( \mathfrak{B} \neq \emptyset \)