This theory defines the maps to study in uniform spaces and proves their basic properties.
Just as the the most general setting for continuity of functions is that of topological spaces, uniform spaces are the most general setting for the study of uniform continuity.
A map between 2 uniformities is uniformly continuous if it preserves the entourages:
definition
\( f:X\rightarrow Y \Longrightarrow \Phi \text{ is a uniformity on } X \Longrightarrow \Gamma \text{ is a uniformity on } Y \Longrightarrow \) \( f \text{ is uniformly continuous between } \Phi \text{ and } \Gamma \equiv \forall V\in \Gamma .\ ( \text{ProdFunction}(f,f)^{-1}V) \in \Phi \)
Any uniformly continuous function is continuous when considering the topologies on the uniformities.
lemma uniformly_cont_is_cont:
assumes \( f:X\rightarrow Y \), \( \Phi \text{ is a uniformity on } X \), \( \Gamma \text{ is a uniformity on } Y \), \( f \text{ is uniformly continuous between } \Phi \text{ and } \Gamma \)
shows \( \text{IsContinuous}( \text{UniformTopology}(\Phi ,X), \text{UniformTopology}(\Gamma ,Y),f) \)proofassumes \( f:X\rightarrow Y \)
shows \( f^{-1}(D) \subseteq X \)assumes \( x\in X \), \( f:X\rightarrow Y \)
shows \( \langle x,t\rangle \in \text{ProdFunction}(f,f)^{-1}(V) \longleftrightarrow t\in X \wedge \langle fx,ft\rangle \in V \)assumes \( f:X\rightarrow Y \)
shows \( f^{-1}(A) = \{x\in X.\ f(x) \in A\} \)