A metric space is a set on which a distance between points is defined as a function \(d:X \times X \to [0,\infty)\). With this definition each metric space is a topological space which is paracompact and Hausdorff (\(T_2\)), hence normal (in fact even perfectly normal).
A metric on \(X\) is usually defined as a function \(d:X \times X \to [0,\infty)\) that satisfies the conditions \(d(x,x) = 0\), \(d(x, y) = 0 \Rightarrow x = y\) (identity of indiscernibles), \(d(x, y) = d(y, x)\) (symmetry) and \(d(x, y) \le d(x, z) + d(z, y)\) (triangle inequality) for all \(x,y \in X\). Here we are going to be a bit more general and define metric and pseudo-metric as a function valued in an ordered loop.
First we define a pseudo-metric, which has the axioms of a metric, but without the second part of the identity of indiscernibles. In our definition IsApseudoMetric is a predicate on five sets: the function \(d\), the set \(X\) on which the metric is defined, the loop carrier \(G\), the loop operation \(A\) and the order \(r\) on \(G\).
definition
\( \text{IsApseudoMetric}(d,X,G,A,r) \equiv d:X\times X \rightarrow \text{Nonnegative}(G,A,r) \) \( \wedge (\forall x\in X.\ d\langle x,x\rangle = \text{ TheNeutralElement}(G,A))\) \( \wedge (\forall x\in X.\ \forall y\in X.\ d\langle x,y\rangle = d\langle y,x\rangle )\) \( \wedge (\forall x\in X.\ \forall y\in X.\ \forall z\in X.\ \langle d\langle x,z\rangle , A\langle d\langle x,y\rangle ,d\langle y,z\rangle \rangle \rangle \in r) \)
We add the full axiom of identity of indiscernibles to the definition of a pseudometric to get the definition of metric.
definition
\( \text{IsAmetric}(d,X,G,A,r) \equiv \) \( \text{IsApseudoMetric}(d,X,G,A,r) \wedge (\forall x\in X.\ \forall y\in X.\ d\langle x,y\rangle = \text{ TheNeutralElement}(G,A) \longrightarrow x=y) \)
A disk is defined as set of points located less than the radius from the center.
definition
\( \text{Disk}(X,d,r,c,R) \equiv \{x\in X.\ \langle d\langle c,x\rangle ,R\rangle \in \text{StrictVersion}(r)\} \)
We define metric topology as consisting of unions of open disks.
definition
\( \text{MetricTopology}(X,L,A,r,d) \equiv \{\bigcup \mathcal{A} .\ \mathcal{A} \in Pow(\bigcup c\in X.\ \{ \text{Disk}(X,d,r,c,R).\ R\in \text{PositiveSet}(L,A,r)\})\} \)
Next we define notation for metric spaces. We will reuse the additive notation defined in the loop1 locale adding only the assumption about \(d\) being a pseudometric and notation for a disk centered at \(c\) with radius \(R\). Since for many theorems it is sufficient to assume the pseudometric axioms we will assume in this context that the sets \(d,X,L,A,r\) form a pseudometric raher than a metric. In the pmetric_space context \(\tau\) denotes the topology defined by the metric \(d\). Analogously to the notation defined in the topology0 context \( int(A) \), \( cl(A) \), \( \partial A \) will denote the interior, closure and boundary of the set \(A\) with respect to the metric topology.
locale pmetric_space = loop1 +
assumes pmetricAssum: \( \text{IsApseudoMetric}(d,X,L,A,r) \)
defines \( disk(c,R) \equiv \text{Disk}(X,d,r,c,R) \)
defines \( \tau \equiv \text{MetricTopology}(X,L,A,r,d) \)
defines \( int(D) \equiv \text{Interior}(D,\tau ) \)
defines \( cl(D) \equiv \text{Closure}(D,\tau ) \)
The next lemma shows the definition of the pseudometric in the notation used in the pmetric_space context.
lemma (in pmetric_space) pmetric_properties:
shows \( d: X\times X \rightarrow L^+ \), \( \forall x\in X.\ d\langle x,x\rangle = 0 \), \( \forall x\in X.\ \forall y\in X.\ d\langle x,y\rangle = d\langle y,x\rangle \), \( \forall x\in X.\ \forall y\in X.\ \forall z\in X.\ d\langle x,z\rangle \leq d\langle x,y\rangle + d\langle y,z\rangle \) using pmetricAssum unfolding IsApseudoMetric_defThe values of the metric are in the in the nonnegative set of the loop, hence in the loop.
lemma (in pmetric_space) pmetric_loop_valued:
assumes \( x\in X \), \( y\in X \)
shows \( d\langle x,y\rangle \in L^+ \), \( d\langle x,y\rangle \in L \)proofThe definition of the disk in the notation used in the pmetric_space context:
lemma (in pmetric_space) disk_definition:
shows \( disk(c,R) = \{x\in X.\ d\langle c,x\rangle \lt R\} \)proofIf the radius is positive then the center is in disk.
lemma (in pmetric_space) center_in_disk:
assumes \( c\in X \) and \( R\in L_+ \)
shows \( c \in disk(c,R) \) using pmetricAssum, assms, IsApseudoMetric_def, PositiveSet_def, disk_definitionA technical lemma that allows us to shorten some proofs: if \(c\) is an element of \(X\) and \(x\) is in disk with center \(c\) and radius \(R\) then \(R\) is a positive element of \(L\) and \(-d(x,y)+R\) is in the set of positive elements of the loop.
lemma (in pmetric_space) radius_in_loop:
assumes \( c\in X \) and \( x \in disk(c,R) \)
shows \( R\in L \), \( 0 \lt R \), \( R\in L_+ \), \( ( - d\langle c,x\rangle + R) \in L_+ \)proofIf a point \(x\) is inside a disk \(B\) and \(m\leq -d\langle c,x\rangle + R\) then the disk centered at the point \(x\) and with radius \(m\) is contained in the disk \(B\).
lemma (in pmetric_space) disk_in_disk:
assumes \( c\in X \) and \( x \in disk(c,R) \) and \( m \leq ( - d\langle c,x\rangle + R) \)
shows \( disk(x,m) \subseteq disk(c,R) \)proofA special case of disk_in_disk where we set \(m = -d\langle c,x\rangle + R\): if \(x\) is an element of a disk with center \(c\in X\) and radius \(R\) then this disk contains the disk centered at \(x\) and with radius \(-d\langle c,x\rangle + R\).
lemma (in pmetric_space) disk_in_disk1:
assumes \( c\in X \) and \( x \in disk(c,R) \)
shows \( disk(x, - d\langle c,x\rangle + R) \subseteq disk(c,R) \)proofAssuming that two disks have the same center, closed disk with smaller radius in contained in the (open) disk with a larger radius.
lemma (in pmetric_space) disk_radius_strict_mono:
assumes \( r_1 \lt r_2 \)
shows \( \{y\in X.\ d\langle x,y\rangle \leq r_1\} \subseteq disk(x,r_2) \) using assms, loop_strict_ord_trans, disk_definitionIf we assume that the loop's order relation down-directs \(L_+\) then the collection of disks centered at points of the space and with radii in the positive set of the loop satisfies the base condition. The property that an order relation "down-directs" a set is defined in Order_ZF and means that every two-element subset of the set has a lower bound in that set.
lemma (in pmetric_space) disks_form_base:
assumes \( r \text{ down-directs } L_+ \)
defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( B \text{ satisfies the base condition } \)proofDisks centered at points farther away than the sum of radii do not overlap.
lemma (in pmetric_space) far_disks:
assumes \( x\in X \), \( y\in X \), \( r_x + r_y \leq d\langle x,y\rangle \)
shows \( disk(x,r_x)\cap disk(y,r_y) = \emptyset \)proofIf we have a loop element that is smaller than the distance between two points, then we can separate these points with disks.
lemma (in pmetric_space) disjoint_disks:
assumes \( x\in X \), \( y\in X \), \( r_x \lt d\langle x,y\rangle \)
shows \( ( - r_x + (d\langle x,y\rangle )) \in L_+ \) and \( disk(x,r_x)\cap disk(y, - r_x + (d\langle x,y\rangle )) = 0 \)proofThe definition of metric topology written in notation of pmetric_space context:
lemma (in pmetric_space) metric_top_def_alt:
defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( \tau = \{\bigcup A.\ A \in Pow(B)\} \)proofIf the order of the loop down-directs its set of positive elements then the metric topology defined as collection of unions of (open) disks is indeed a topology. Recall that in the pmetric_space context \(\tau\) denotes the metric topology.
theorem (in pmetric_space) pmetric_is_top:
assumes \( r \text{ down-directs } L_+ \)
shows \( \tau \text{ is a topology } \) using assms, disks_form_base, Top_1_2_T1, metric_top_def_altIf \(r\) down-directs \(L_+\) then the collection of open disks is a base for the metric topology.
theorem (in pmetric_space) disks_are_base:
assumes \( r \text{ down-directs } L_+ \)
defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( B \text{ is a base for } \tau \) using assms, disks_form_base, Top_1_2_T1, metric_top_def_altIf \(r\) down-directs \(L_+\) then \(X\) is the carrier of metric topology.
theorem (in pmetric_space) metric_top_carrier:
assumes \( r \text{ down-directs } L_+ \)
shows \( \bigcup \tau = X \)proofUnder the assumption that \(r\) down-directs \(L_+\) the propositions proven in the topology0 context can be used in the pmetric_space context.
lemma (in pmetric_space) topology0_valid_in_pmetric_space:
assumes \( r \text{ down-directs } L_+ \)
shows \( topology0(\tau ) \) using assms, pmetric_is_top unfolding topology0_defIf \(r\) down-directs \(L_+\) then disks are open in the metric topology.
lemma (in pmetric_space) disks_open:
assumes \( c\in X \), \( R\in L_+ \), \( r \text{ down-directs } L_+ \)
shows \( disk(c,R) \in \tau \) using assms, base_sets_open, disks_are_base(1), pmetric_is_topTo define the metric_space locale we take the pmetric_space and add the assumption of identity of indiscernibles.
locale metric_space = pmetric_space +
assumes ident_indisc: \( \forall x\in X.\ \forall y\in X.\ d\langle x,y\rangle = 0 \longrightarrow x=y \)
In the metric_space locale \(d\) is a metric.
lemma (in metric_space) d_metric:
shows \( \text{IsAmetric}(d,X,L,A,r) \) using pmetricAssum, ident_indisc unfolding IsAmetric_defDistance of different points is greater than zero.
lemma (in metric_space) dist_pos:
assumes \( x\in X \), \( y\in X \), \( x\neq y \)
shows \( 0 \lt d\langle x,y\rangle \), \( d\langle x,y\rangle \in L_+ \)proofIf \(r\) down-directs \(L_+\) then the ordered loop valued metric space is \(T_2\) (i.e. Hausdorff).
theorem (in metric_space) metric_space_T2:
assumes \( r \text{ down-directs } L_+ \)
shows \( \tau \text{ is }T_2 \)proofEach pseudometric space with pseudometric \(d:X\times X\rightarrow L\) supports a natural uniform structure, defined as supersets of the collection of inverse images \(U_c = d^{-1}([0,c])\), where \(c>0\).
In the following definition \(X\) is the underlying space, \(L\) is the loop (carrier), \(A\) is the loop operation, \(r\) is an order relation compatible with \(A\), and \(d\) is a pseudometric on \(X\), valued in the ordered loop \(L\). With this we define the uniform gauge as the collection of inverse images of the closed intervals \([0,c]\) as \(c\) varies of the set of positive elements of \(L\).
definition
\( \text{UniformGauge}(X,L,A,r,d) \equiv \{d^{-1}(\{b\in \text{Nonnegative}(L,A,r).\ \langle b,c\rangle \in r\}).\ c\in \text{PositiveSet}(L,A,r)\} \)
In the pmetric_space context we will write \( \text{UniformGauge}(X,L,A,r,d) \) as \( \mathfrak{B} \).
abbreviation (in pmetric_space)
\( \mathfrak{B} \equiv \text{UniformGauge}(X,L,A,r,d) \)
In notation defined in the pmetric_space context we can write the uniform gauge as \(\{ d^{-1}(\{c\in L^+: c\leq b\}: b \in L_+ \}\).
lemma (in pmetric_space) uniform_gauge_def_alt:
shows \( \mathfrak{B} = \{d^{-1}(\{c\in L^+.\ c\leq b\}).\ b\in L_+\} \) unfolding UniformGauge_defMembers of the uniform gauge are subsets of \(X\times X\) i.e. relations on \(X\).
lemma (in pmetric_space) uniform_gauge_relations:
assumes \( B\in \mathfrak{B} \)
shows \( B\subseteq X\times X \) using assms, uniform_gauge_def_alt, pmetric_properties(1), func1_1_L3If the distance between two points of \(X\) is less or equal \(b\), then this pair of points is in \(d^{-1}([0,b])\).
lemma (in pmetric_space) gauge_members:
assumes \( x\in X \), \( y\in X \), \( d\langle x,y\rangle \leq b \)
shows \( \langle x,y\rangle \in d^{-1}(\{c\in L^+.\ c\leq b\}) \) using assms, pmetric_properties(1), apply_funtype, func1_1_L15Suppose \(b\in L^+\) (i.e. b is an element of the loop that is greater than the neutral element) and \(x\in X\). Then the image of the singleton set \(\{ x\}\) by the relation \(B=\{ d^{-1}(\{c\in L^+: c\leq b\}\) is the set \(\{ y\in X:d\langle x,y\rangle \leq b\}\), i.e. the closed disk with center \(x\) and radius \(b\). Hence the the image \(B\{ x\}\) contains the open disk with center \(x\) and radius \(b\).
lemma (in pmetric_space) disk_in_gauge:
assumes \( b\in L_+ \), \( x\in X \)
defines \( B \equiv d^{-1}(\{c\in L^+.\ c\leq b\}) \)
shows \( B\{x\} = \{y\in X.\ d\langle x,y\rangle \leq b\} \) and \( disk(x,b) \subseteq B\{x\} \)proofGauges corresponding to larger elements of the loop are larger.
lemma (in pmetric_space) uniform_gauge_mono:
assumes \( b_1\leq b_2 \)
shows \( d^{-1}(\{c\in L^+.\ c\leq b_1\}) \subseteq d^{-1}(\{c\in L^+.\ c\leq b_2\}) \) using ordLoopAssum, assms, vimage_mono1 unfolding IsAnOrdLoop_def, IsPartOrder_def, trans_defFor any two sets of the form \(d^{-1}([0,b])\) we can find a third one that is contained in both.
lemma (in pmetric_space) gauge_1st_cond:
assumes \( r \text{ down-directs } L_+ \), \( B_1\in \mathfrak{B} \), \( B_2\in \mathfrak{B} \)
shows \( \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \)proofSets of the form \(d^{-1}([0,b])\) contain the diagonal.
lemma (in pmetric_space) gauge_2nd_cond:
assumes \( B\in \mathfrak{B} \)
shows \( id(X)\subseteq B \)proofSets of the form \(d^{-1}([0,b])\) are symmetric.
lemma (in pmetric_space) gauge_symmetric:
assumes \( B\in \mathfrak{B} \)
shows \( B = converse(B) \)proofA set of the form \(d^{-1}([0,b])\) contains a symmetric set of this form.
corollary (in pmetric_space) gauge_3rd_cond:
assumes \( B_1\in \mathfrak{B} \)
shows \( \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \) using assms, gauge_symmetricThe collection of sets of the form \(d^{-1}([0,b])\) for \(b\in L_+\) is contained of the powerset of \(X\times X\).
lemma (in pmetric_space) gauge_5thCond:
shows \( \mathfrak{B} \subseteq Pow(X\times X) \) using uniform_gauge_def_alt, pmetric_properties(1), func1_1_L3If the set of positive values is non-empty, then there are sets of the form \(d^{-1}([0,b])\) for \(b>0\).
lemma (in pmetric_space) gauge_6thCond:
assumes \( L_+\neq \emptyset \)
shows \( \mathfrak{B} \neq \emptyset \) using assms, uniform_gauge_def_altThe remaining 4th condition for the sets of the form \(d^{-1}([0,b])\) to be a uniform base (or a fundamental system of entourages) cannot be proven without additional assumptions in the context of ordered loop valued metrics. To see that consider the example of natural numbers with the metric \(d\langle x,y \rangle = |x-y|\), where we think of \(d\) as valued in the nonnegative set of ordered group of integers. Now take the set \(B_1 = d^{-1}([0,1]) = d^{-1}(\{ 0,1\} )\). Then the set \(B_1 \circ B_1\) is strictly larger than \(B_1\), but there is no smaller set \(B_2\) we can take so that \(B_2 \circ B_2 \subseteq B_1\). One condition that is sufficient is that for every \(b_1 >0\) there is a \(b_2 >0\) such that \(b_2 + b_2 \leq b_1 \). I have not found a standard name for this property, for now we will use the name IsHalfable.
definition
\( \text{IsHalfable}(L,A,r) \equiv \forall b_1\in \text{PositiveSet}(L,A,r).\ \exists b_2\in \text{PositiveSet}(L,A,r).\ \langle A\langle b_2,b_2\rangle ,b_1\rangle \in r \)
The property of halfability written in the notation used in the pmetric_space context.
lemma (in pmetric_space) is_halfable_def_alt:
assumes \( \text{IsHalfable}(L,A,r) \), \( b_1\in L_+ \)
shows \( \exists b_2\in L_+.\ b_2 + b_2 \leq b_1 \) using assms unfolding IsHalfable_defIf the loop order is halfable then for every set \(B_1\) of the form \(d^{-1}([0,b_1])\) for some \(b_1>0\) we can find another one \(B_2 = d^{-1}([0,b_2])\) such that \(B_2\) composed with itself is contained in \(B_1\).
lemma (in pmetric_space) gauge_4thCond:
assumes \( \text{IsHalfable}(L,A,r) \), \( B_1\in \mathfrak{B} \)
shows \( \exists B_2\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \)proofIf \(X\) and \(L_+\) are not empty, the order relation \(r\) down-directs \(L_+\), and the loop order is halfable, then \(\mathfrak{B}\) (which in the pmetric_space context is an abbreviation for \(\{ d^{-1}(\{c\in L^+: c\leq b\}: b \in L_+ \}\)) is a fundamental system of entourages, hence its supersets form a uniformity on \(X\) and hence those supersets define a topology on \(X\).
theorem (in pmetric_space) metric_gauge_base:
assumes \( X\neq \emptyset \), \( L_+\neq \emptyset \), \( r \text{ down-directs } L_+ \), \( \text{IsHalfable}(L,A,r) \)
shows \( \mathfrak{B} \text{ is a uniform base on } X \), \( \text{Supersets}(X\times X,\mathfrak{B} ) \text{ is a uniformity on } X \), \( \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) \text{ is a topology } \), \( \bigcup \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) = X \) using assms, gauge_1st_cond, gauge_2nd_cond, gauge_3rd_cond, gauge_4thCond, gauge_5thCond, gauge_6thCond, uniformity_base_is_base, uniform_top_is_top unfolding IsUniformityBaseOn_defAt this point we know that a pseudometric induces two topologies: one consisting of unions of open disks (the metric topology) and second one being the uniform topology derived from the uniformity generated the fundamental system of entourages (the base uniformity) of the sets of the form \(d^{-1}([0,b])\) for \(b>0\). The next theorem states that if \(X\) and \(L_+\) are not empty, \(r\) down-directs \(L_+\), and the loop order is halfable, then these two topologies are in fact the same. Recall that in the pmetric_space context \(\tau\) denotes the metric topology.
theorem (in pmetric_space) metric_top_is_uniform_top:
assumes \( X\neq \emptyset \), \( L_+\neq \emptyset \), \( r \text{ down-directs } L_+ \), \( \text{IsHalfable}(L,A,r) \)
shows \( \tau = \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) \)proofassumes \( x\leq y \) and \( y \lt z \)
shows \( x \lt z \)assumes \( x \lt y \)
shows \( 0 \lt - x + y \), \( ( - x + y) \in L_+ \), \( 0 \lt y - x \), \( (y - x) \in L_+ \)assumes \( c\in X \) and \( x \in disk(c,R) \)
shows \( R\in L \), \( 0 \lt R \), \( R\in L_+ \), \( ( - d\langle c,x\rangle + R) \in L_+ \)assumes \( x \lt y \) and \( y\leq z \)
shows \( x \lt z \)assumes \( x \lt y \), \( z\in L \)
shows \( x + z \lt y + z \) and \( z + x \lt z + y \)assumes \( x\in G \), \( y\in G \)
shows \( \exists !z.\ z\in G \wedge z\cdot x = y \), \( y/ x \in G \), \( (y/ x)\cdot x = y \) and \( \exists !z.\ z\in G \wedge x\cdot z = y \), \( x\backslash y \in G \), \( x\cdot (x\backslash y) = y \)assumes \( x \lt y \)
shows \( x\in L \) and \( y\in L \)assumes \( x\in L \), \( y\in L \)
shows \( ( - x + y) \in L \) and \( x - y \in L \)assumes \( x\in L \)
shows \( x\leq x \)assumes \( c\in X \) and \( x \in disk(c,R) \) and \( m \leq ( - d\langle c,x\rangle + R) \)
shows \( disk(x,m) \subseteq disk(c,R) \)assumes \( c\in X \) and \( x \in disk(c,R) \)
shows \( R\in L \), \( 0 \lt R \), \( R\in L_+ \), \( ( - d\langle c,x\rangle + R) \in L_+ \)assumes \( c\in X \) and \( R\in L_+ \)
shows \( c \in disk(c,R) \)assumes \( x \lt y \), \( z \lt t \)
shows \( x + z \lt y + t \)assumes \( x \lt y \)
shows \( 0 \lt - x + y \), \( ( - x + y) \in L_+ \), \( 0 \lt y - x \), \( (y - x) \in L_+ \)assumes \( x \lt y \)
shows \( x\in L \) and \( y\in L \)assumes \( x\in X \), \( y\in X \)
shows \( d\langle x,y\rangle \in L^+ \), \( d\langle x,y\rangle \in L \)assumes \( x\in X \), \( y\in X \), \( r_x + r_y \leq d\langle x,y\rangle \)
shows \( disk(x,r_x)\cap disk(y,r_y) = \emptyset \)assumes \( r \text{ down-directs } L_+ \)
defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( B \text{ satisfies the base condition } \)assumes \( B \text{ satisfies the base condition } \) and \( T = \{\bigcup A.\ A\in Pow(B)\} \)
shows \( T \text{ is a topology } \) and \( B \text{ is a base for } T \)defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( \tau = \{\bigcup A.\ A \in Pow(B)\} \)assumes \( r \text{ down-directs } L_+ \)
defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( B \text{ is a base for } \tau \)assumes \( B \text{ is a base for } T \)
shows \( \bigcup T = \bigcup B \)assumes \( r \text{ down-directs } L_+ \)
shows \( \tau \text{ is a topology } \)assumes \( B \text{ is a base for } T \) and \( U \in B \)
shows \( U \in T \)assumes \( r \text{ down-directs } L_+ \)
defines \( B \equiv \bigcup c\in X.\ \{disk(c,R).\ R\in L_+\} \)
shows \( B \text{ is a base for } \tau \)assumes \( r \text{ down-directs } L_+ \)
shows \( \bigcup \tau = X \)assumes \( x\in X \), \( y\in X \), \( x\neq y \)
shows \( 0 \lt d\langle x,y\rangle \), \( d\langle x,y\rangle \in L_+ \)assumes \( x \lt y \)
shows \( 0 \lt - x + y \), \( ( - x + y) \in L_+ \), \( 0 \lt y - x \), \( (y - x) \in L_+ \)assumes \( x\in X \), \( y\in X \)
shows \( d\langle x,y\rangle \in L^+ \), \( d\langle x,y\rangle \in L \)assumes \( x\in X \), \( y\in X \), \( x\neq y \)
shows \( 0 \lt d\langle x,y\rangle \), \( d\langle x,y\rangle \in L_+ \)assumes \( x\in L \), \( 0 \lt y \)
shows \( x - y \lt x \), \( ( - y + x) \lt x \), \( x \lt x + y \), \( x \lt y + x \)assumes \( x\in X \), \( y\in X \), \( r_x \lt d\langle x,y\rangle \)
shows \( ( - r_x + (d\langle x,y\rangle )) \in L_+ \) and \( disk(x,r_x)\cap disk(y, - r_x + (d\langle x,y\rangle )) = 0 \)assumes \( A\subseteq B \) and \( \exists x\in A.\ \exists y\in A.\ \phi (x,y) \)
shows \( \exists x\in B.\ \exists y\in B.\ \phi (x,y) \)assumes \( f:X\rightarrow Y \)
shows \( f^{-1}(D) \subseteq X \)assumes \( f:X\rightarrow Y \)
shows \( f^{-1}(A) = \{x\in X.\ f(x) \in A\} \)assumes \( B\in \mathfrak{B} \)
shows \( B\subseteq X\times X \)assumes \( A\subseteq B \)
shows \( f^{-1}(A) \subseteq f^{-1}(B) \)assumes \( b_1\leq b_2 \)
shows \( d^{-1}(\{c\in L^+.\ c\leq b_1\}) \subseteq d^{-1}(\{c\in L^+.\ c\leq b_2\}) \)assumes \( f:X\times X\rightarrow Y \) and \( \forall x\in X.\ \forall y\in X.\ f\langle x,y\rangle = f\langle y,x\rangle \)
shows \( f^{-1}(A) = converse(f^{-1}(A)) \)assumes \( B\in \mathfrak{B} \)
shows \( B = converse(B) \)assumes \( \text{IsHalfable}(L,A,r) \), \( b_1\in L_+ \)
shows \( \exists b_2\in L_+.\ b_2 + b_2 \leq b_1 \)assumes \( x\leq y \), \( z\leq t \)
shows \( x + z \leq y + t \)assumes \( x\leq y \) and \( y\leq z \)
shows \( x\leq z \)assumes \( x\in X \), \( y\in X \), \( d\langle x,y\rangle \leq b \)
shows \( \langle x,y\rangle \in d^{-1}(\{c\in L^+.\ c\leq b\}) \)assumes \( r \text{ down-directs } L_+ \), \( B_1\in \mathfrak{B} \), \( B_2\in \mathfrak{B} \)
shows \( \exists B_3\in \mathfrak{B} .\ B_3\subseteq B_1\cap B_2 \)assumes \( B\in \mathfrak{B} \)
shows \( id(X)\subseteq B \)assumes \( B_1\in \mathfrak{B} \)
shows \( \exists B_2\in \mathfrak{B} .\ B_2 \subseteq converse(B_1) \)assumes \( \text{IsHalfable}(L,A,r) \), \( B_1\in \mathfrak{B} \)
shows \( \exists B_2\in \mathfrak{B} .\ \exists B_2\in \mathfrak{B} .\ B_2\circ B_2 \subseteq B_1 \)assumes \( L_+\neq \emptyset \)
shows \( \mathfrak{B} \neq \emptyset \)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 \)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\neq \emptyset \), \( L_+\neq \emptyset \), \( r \text{ down-directs } L_+ \), \( \text{IsHalfable}(L,A,r) \)
shows \( \mathfrak{B} \text{ is a uniform base on } X \), \( \text{Supersets}(X\times X,\mathfrak{B} ) \text{ is a uniformity on } X \), \( \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) \text{ is a topology } \), \( \bigcup \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) = X \)assumes \( X\neq \emptyset \), \( L_+\neq \emptyset \), \( r \text{ down-directs } L_+ \), \( \text{IsHalfable}(L,A,r) \)
shows \( \mathfrak{B} \text{ is a uniform base on } X \), \( \text{Supersets}(X\times X,\mathfrak{B} ) \text{ is a uniformity on } X \), \( \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) \text{ is a topology } \), \( \bigcup \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) = X \)assumes \( b\in L_+ \), \( x\in X \)
defines \( B \equiv d^{-1}(\{c\in L^+.\ c\leq b\}) \)
shows \( B\{x\} = \{y\in X.\ d\langle x,y\rangle \leq b\} \) and \( disk(x,b) \subseteq B\{x\} \)assumes \( c\in X \), \( R\in L_+ \), \( r \text{ down-directs } L_+ \)
shows \( disk(c,R) \in \tau \)assumes \( r \text{ down-directs } L_+ \)
shows \( topology0(\tau ) \)assumes \( \forall x\in V.\ \exists U\in T.\ (x\in U \wedge U\subseteq V) \)
shows \( V\in T \)assumes \( c\in X \) and \( x \in disk(c,R) \)
shows \( disk(x, - d\langle c,x\rangle + R) \subseteq disk(c,R) \)assumes \( x\in L \), \( 0 \lt y \)
shows \( x - y \lt x \), \( ( - y + x) \lt x \), \( x \lt x + y \), \( x \lt y + x \)assumes \( r_1 \lt r_2 \)
shows \( \{y\in X.\ d\langle x,y\rangle \leq r_1\} \subseteq disk(x,r_2) \)assumes \( A\subseteq X \), \( A\in \mathcal{A} \)
shows \( A \in \text{Supersets}(X,\mathcal{A} ) \)assumes \( b\in L_+ \), \( x\in X \)
defines \( B \equiv d^{-1}(\{c\in L^+.\ c\leq b\}) \)
shows \( B\{x\} = \{y\in X.\ d\langle x,y\rangle \leq b\} \) and \( disk(x,b) \subseteq B\{x\} \)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\} \)assumes \( X\neq \emptyset \), \( L_+\neq \emptyset \), \( r \text{ down-directs } L_+ \), \( \text{IsHalfable}(L,A,r) \)
shows \( \mathfrak{B} \text{ is a uniform base on } X \), \( \text{Supersets}(X\times X,\mathfrak{B} ) \text{ is a uniformity on } X \), \( \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) \text{ is a topology } \), \( \bigcup \text{UniformTopology}( \text{Supersets}(X\times X,\mathfrak{B} ),X) = X \)assumes \( B \text{ is a base for } T \) and \( S \text{ is a topology } \) and \( B\subseteq S \)
shows \( T\subseteq S \)