Some Cursory Notes - LATEX
Some Cursory Notes - LATEX
METRIC SPACES
1. d(x, y) = 0 ⇐⇒ x = y (Positivity)
1
2 Metric Spaces
Theorem 1.6
Convergence =⇒ cauchy
3. ⟨u|u⟩ > 0 if u ̸= 0
We say dp (⃗x, ⃗y ), the distance between ⃗x and ⃗y to be ||x − y||p = ( ni=1 |xi − yi |p )1/p . From
P
this definition, unique 0 distance P property and reflexivity property are obvious. Consider
dp (x, z) and dp (z, y). dp (x, y) = ( ki=1 |(xi − zi ) + (zi − yi )|p )1/p whence from Minkowski
we see that
k
X Xn n
X
( |(xi − zi ) + (zi − yi )|p )1/p ≤ ( |xi − zi |p )1/p + ( |zi − yi |p )1/p = dp (x, z) + dp (y, z)
i=1 i=1 i=1
This is a metric due to positive definiteness and symmetry. The triangle inequality is,
also, not hard to see. ■
Example : Space of all bounded sequences
Let X be the set of all bounded sequences of reals, i.e, the set of all x such that x =
(x1 , x2 , · · · ) = {xn }∞ n
n=1 with supi=1 ({xi }) < ∞. If {xi } and {yi } are sequences (i,e,
elements in X) let the distance between two sequences be defined by
∞
d(x, y) := sup |xi − yi |
i=1
Clearly, it is positive definite and symmetric. Consider three sequences {xn }, {yn } and
{zn } in X. d(x, y) = sup{|xi − yi | : i ∈ N}, d(x, z) = sup{|xi − zi | : i ∈ N} and
d(y, z) = sup{|yi − zi | : i ∈ N}. Cosnider d(x, z) = sup{|xi − zi | = |xi − yi + yi − zi | : i ∈
N} ≤ sup{|xi − yi | + |yi − zi | : i ∈ N} =⇒ ≤ sup{|xi − yi | : i ∈ N} + sup{|yi − zi | : i ∈ N}
which proves the triangle. ■
Metric Spaces 5
(∀ε > 0)(∃δ > 0)(∀p ∈ X)(dx (p, a) < δ =⇒ dy (f (p), f (a)) < ε)
Corollary 1.11
Composition of continuous functions (at a point a) is finally a continuous function
to f (a). From the continuity of g, we note that g ◦ (f (xn )) converges to g ◦ (f (a)), which
ultimately tells that for every sequence {xn } in X that converges to a, g ◦ f (xn ) is a
sequence in Z that converges to g ◦ f (a) whence we are done ■
Example : Dirichlet Function
Let f : R → R be defined by
(
1 if x is rational
f (x) =
0 if x is irrational
This function is discontinuous at every point of R. Bear in mind that to show that a
function is discontinuous at a point z, we need only show that one sequence in A which
converges to z is such that lim(f (xn )) ̸= f (lim(xn )). Consider a ∈ R an irrational point.
Consider the rational sequence xn that converges to a via density theorem. f (xn ) = 1 for
every n ∈ N which means lim f (xn ) = 1. But f (lim(xn )) = 0. Hence, discontinuous at
a ∈ R, irrational. In fact, the same argument can be re-used to show that f is irrational
at every point. ■
Example : Thomae Function
We define the Thomae function as follows: Let f : R+ → R,
(
0 if x is irrational
f (x) :=
1/n if x is rational, with x = m/n, gcd(m, n) = 1
This function is discontinuous at rational points quite obviously since, consider a rational
number m/n where f (m/n) = 1/n > 0. Consider an irrational sequence in R+ converging
to m/n. Clearly, f (xn ) = 0 for every n ∈ N whence, it is clear.
f (bn ) > 0. From Nested interval theorem, we have γ ∈ ∩n [an , bn ], moreover, since the size
of these intervals are converging to 0, this is a unique point in the intersection. an → γ
and bn → γ. From continuity, then, we have f (an ) → f (γ) ≤ 0 and f (bn ) → f (γ) ≥ 0
which means that f (γ) = 0. ■
Let a < b and define g(x) = f (x) − k. This is a continuous mapping on I. We then have
g(a) < 0 < g(b) whence from location or roots theorem, we find c ∈ I so that g(c) = 0 or
f (c) = k. ■
Consider f (I) := {z ∈ R : ∃x ∈ I such that f (x) = z}. We know that continuous functions
attain bounds, i.e, f (I) has a maxima and a minima that will (eventually) be the end points
of our closed bounded interval. If the function is constant, we are done. Consider a point
min(f (I)) < z < max(f (I)). By Bolzano’s IVT, we know that a pre-image exists for z.
This means that z is in the image. We are, therefore, done. The requisite interval is
[min(f ), max(f )]. ■
Theorem 1.18
Let f be a function defined on A ⊆ R. The following are equivalent:
2. ∃ε > 0 such that ∀δ > 0, ∃xδ , uδ ∈ A so that 0 < |xδ − uδ | < δ but |f (xδ ) −
f (uδ )| ≥ ε
(2) =⇒ (3)) Choose δ = 1, and get corresponding x1 , u1 so that 0 < |x1 − u1 | < 1
and |f (x1 ) − f (u1 )| ≥ ε. Choose δ = 1/2 and get the corresponding x2 and u2 so that
0 < |x2 − u2 | < 1/2 and |f (x2 ) − f (u2 )| ≥ ε. Keep going as such to get xn , un so that
0 < |xn − un | < 1/n ∀n ∈ N and |f (xn ) − f (un )| ≥ ε for every n ∈ N. This means that
lim(xn − un ) = 0 but |f (xn ) − f (un )| ≥ ε for every n ∈ N.
(3) =⇒ (2)) ∀δ > 0, ∃n0 (δ) so that ∀n ≥ n0 , we have 0 < |xn − un | < δ but
|f (xn ) − f (un )| ≥ ε , choose one of these xn −s for n greater than n0 (δ) as our xδ (and
likewise for uδ ). We are then done. ■
Sequences of Functions
Given a set A ⊂ R, we primarily work with a (countably) infinite collection of functions
{fn } with fn : A → R. We generate a sequence of numbers by evaluating fn at a fixed
point x ∈ A. It could be, then, that {fn (x)}, treated as a sequence of numbers in R, either
converges or does not. For a subset A0 ⊆ A (which can possibly be empty), fn (x) converges
10 Metric Spaces
for every x ∈ A0 . If this happens, there is a uniquely determined value that we would like to
call "f (x)". Thus, there arises naturally a function f : A0 → R that we call the "limit" of
{fn }.
Obvious ■
Metric Spaces 11
||ϕ||A := sup{|ϕ(x)| : x ∈ A}
Lemma 1.24
A sequence fn of bounded functions on A converges uniformly to f : A → R if and
only if ||fn − f ||A → 0
Suppose that ∀ε > 0, ∃n0 ∈ N so that ∀m, n ≥ n0 , ||fm − fn ||A ≤ ε which means
that for every x ∈ A, we have |fm (x) − fn (x)| < ε. This means that for every x, fn (x) is
a cauchy sequence, hence convergent to some f (x). More can be said for the sequence at
each x. Fix some x ∈ A. We have that ∀ε > 0, ∃n0 (ε) ∈ N so that ∀n, m ≥ n0 , we have
|fn (x) − fm (x)| < ε which means that ∀n ≥ n0 , |fn (x) − f (x)| < ε which means that, all
in all, ∀ε > 0, ∃n0 (ε) ∈ N so that ∀n ≥ n0 , ∀x ∈ A, we have |fn (x) − f (x)| < ε which is
12 Metric Spaces
lp Space
PIt is easily seen thet lp is a vector space over R. We defne the metric on lp as dp ({x}, {y}) =
( ∞i=1 |x i − y i |p 1/p
) . Positive definiteness is clear since the sum would not be 0 if even one
index is different. Symmetry is obvious, and triangle:
∞
X ∞
X
d(x, z) = ( |xi − zi |p )1/p ≤ ( |xi − yi + yi − zi |p )1/p
i=1 i=1
which gives
∞
X ∞
X
p 1/p
≤( |xi − yi | ) +( |yi − zi |p )1/p = d(x, y) + d(y, z)
i=1 i=1
2. ||αx|| = |α|||x||
1. d(x, y) ≥ 0
2. d(x, y) = 0
3. d(x, y) = d(y, z)
The part that is different is that, for metric spaces, we require that if the distance is 0,
the points are the same. But for psuedometric spaces, the points can be different yet
of the same distance.
Suppose a sequence x⃗k converges to ⃗x, i.e, (xk1 , xk2 · · · xkn ) → (x1 , x2 , · · · xn ). This means
that for every ε > 0, there exists a n0 ∈ N so that ∀k ∈ N, k ≥ n0 would mean that
n
X
( (|xki − xi |p ))1/p < ε
i=1
Suppose that limk→∞ xkj = xj for every j ≤ n, i.e, coordinate wise convergence. That
means that for a given j,for every ε > 0, there exists n0 (ε, j) such that ∀k ∈ N, k ≥ n0 (ε, j)
ε
means that |xkj − xj | < n1/p . If we take the maximum of all the n0 (ε, j), and sum
εp 1/p
Pn k p 1/p n
= ε, which implies convergence in Rn . In a simi-
P
( i=1 |xj − xj | ) = i=1 ( n )
n
lar fashion, we can show that R , d∞ , the max norm, has equivalence between convergence
and coordinate wise convergence ■
Theorem 1.30
Rn with the metric d∞ (x, y) = max{|xj − yj | : j ≤ n} also has an equivalence between
convergence and coordinate wise convergence.
. Is this sequence cauchy? Yes. Consider [0,1] |fm (x) − fn (x)|dx ≤ 21 (n + m/(mn)). For
R
any given ε, we can make m, n large enough to go below it. Suppose that fn converges
to some f , implying that for every R x ∈ [0, 1], we have that ∀ε, ∃n0 ∈ R N so that ∀n ∈
N, n ≥ n0 implies d(fn , f ) = [0,1] |fn (x) − f (x)| < ε. d(fn , f ) = [0, 1 − 1 ] |f (x)|dx +
R R 2 n
1 1 |fn (x) − f (x)|dx + |1 − f (x)|dx but since limn→∞ (d(fn , f )) → 0, we require
[ 21 − n ,2] [ 12 ,1]
R R
that [0, 1 − 1 ] |f (x)|dx = 0 and [ 1 ,1] |1 − f (x)|dx = 0. Since f is continuous (or supposed
2 n 2
to be), we see that f (x) = 0 from 0 to 12 , but 1 from 1
2
to 1, which is absurd. ■
Theorem 1.33
R with d(x, y) = |x − y| is a complete metric space
Theorem 1.34
Rn with dp , d∞ , is complete.
Theorem 1.35
ℓp space, space of all p- summable sequences in R, is a complete metric space.
for all a, b ≥ n0 , (for every j, too). We take the b → ∞ limit here, to get:
j
X
( |xai − xi |p )1/p < ε
i=1
for all a ≥ n0 and ∀j. From monotone convergence theorem, we can take the j limit as
well, to arrive at: ∀ε, ∃n0 so that ∀a ≥ n0 , we have
X∞
a
dp (x , x)( |xai − xi |p )1/p < ε
i=1
which lets us conclude xk → x. But the question is, is x ∈ ℓp ? Consider ( ji=1 |xi |p )1/p ≤
P
( ji=1 |xai − xi |p )1/p + ( ji=1 |xai |p )1/p (Minkowski). Both the summands on the right side
P P
are convergent (by MCT, and definition, respectively). Hence x ∈ ℓp , which makes ℓp a
complete space ■
Theorem 1.36
Set of all bounded sequences on R with d∞ norm is complete
Theorem 1.37
Set C[0, 1] of all continuous functions on closed, bounded interval [0, 1] is cauchy com-
plete under the supremum norm.
Let ε > 0 be arbitrary. For every function fn , there exists δ(n)(ε) > 0 so that ∀a, b ∈ [0, 1],
0 < |a − b| < δ =⇒ |fn (a) − fn (b)| < ε/4. We also note that, there exists an n0 so that
for all m, n > n0 , we have for every x ∈ [0, 1], |fn (x) − fm (x)| < ε/4 for all m, n ≥ n0 .
Moreover, we also have that there exists n′ ∈ N so that |fn (x) − f (x)| < ε/4 for all x,
∀n ≥ n′ .
|f (a) − f (b)| = |f (a) − fn (a) + fn (a) − fm (a) + fm (a) − fm (b) + fm (b) − f (b)| ≤ |fn (a) −
f (a)|+|fm (a)−fm (b)|+|fn (a)−fm (a)|+|fm (b)−f (b)| There exists δ, minimum of the two
δn , δm that ensures that the first two modulii go lower than ε/4. There exists large enough
m, n to ensure the remaining terms go lower than ε/4 as well. All together, we have that
∃δ > 0 so that if a, b ∈ [0, 1] such that 0 < |a − b| < δ, we have |f (a) − f (b)| < 4(ε/4) = ε.
Hence, f is continuous. Therefore, C[0, 1] (and more generally, C[I]) is complete. ■
18 Metric Spaces
In other words, in every ε-ball around p, there would exist a point qε in E, which is
different from p.
Theorem 1.39
Every ball / neighbourhood of p which is a limit point of E, would contain infinitely
many points q such that q ∈ Bε (p) ∩ E \ {p}
Suppose for some neighbourhood, there only exists finite points q1 , q2 , · · · qk such that
qj ∈ Bε0 ∪ E \ {p}. Let δ < min{d(p, qj ) : j ∈ [1, 2, ...k]}. We then have that, there exists
no point q ∈ E such that its distancce from p is less than δ, making p a non-limit point.
Absurd. ■
Corollary 1.40
A finite set has no limit points
⇐= ) Suppose there is a sequence xn such that xn ̸= p∀n ∈ N and ∀ε, ∃n0 (ε) such
that ∀n ≥ n0 we have d(xn , p) < ε which means for a given ε, there exists a point xn0 +1
in E such that it is not equal to p and it is in the ε-ball of p. Hence, p would be a limit
point. ■
Metric Spaces 19
Theorem 1.45
Every open ball is an open set
E C := {x ∈ X : x ̸∈ E}
Consider (∪α Eα )c = {x ∈ X : ∃α ∈ A : x ∈ Eα }c = {x ∈ X : ∀α ∈ A : x ̸∈ Eα } = {x ∈
X : ∀α ∈ A : x ∈ Eαc } = ∩α Eαc ■
⇐= ) Suppose E is closed but E c is not open. This means that there is a point in
E c , p, such that for every ε-ball around p, some point in E falls into this ball. But this
makes p a limit point of E, which is absurd since E is closed, limit points fall into the sets
themselves. ■
Theorem 1.50
For a collection of open sets {Gα : α ∈ A}, ∪α Gα is also an open set.
Corollary 1.51
For any collection of closed sets Eα , ∩α Eα is also closed.
Theorem 1.52
For any finite collection of open sets {E1 , E2 , · · · Ek }, ∩ki=1 Ei is also open.
Corollary 1.53
For any finite collection of closed sets {G1 , G2 , · · · Gk } we have ∪kj=1 Gj to be closed
Remark.
In the above theorem and corollary, we require that the collection be finite. The reason
is that, we were able to get a minimal εj in the proof due to the finiteness of the set. It
may not be possible to find a number δ that is both larger than 0 but smaller than a given
infinite collection of ε-s. For example, consider the sequence of open sets (− n1 , n1 ). The
infinite intersection of these yields {0} which is a closed set by virtue of being finite.
Ē := E ∪ E ′
Theorem 1.56
Closure of a set is closed
or
∃δ(ε) > 0 such that ∃rδ ∈ E such that rδ ̸= p and rδ ∈ Bε (p). In either case, there
would exist a point dependent on ε, in E such that the point itself is different from p, and
exists in the ε-ball around p. Hence, we see that p is a limit point of E. Therefore, we see
that all the limit points of E either are points of E or points of E ′ . Hence, Ē is closed.
■
Theorem 1.57
Ē = E ⇐⇒ E is closed
⇐= ) if E is closed, E ′ ⊆ E =⇒ E ′ ∪ E = E = Ē ■
Fact 1.59
Topological Definition for Closure: The closure of A ⊆ X, denoted by A is defined as
the smallest closed set that contains A
Ā := {x ∈ X : ∀ε > 0, Bε (x) ∩ A ̸= ϕ}
Remark.
A set which is open relative to Y need not be open relative to X. For example, consider
R as a subset of Rn . An interval in R is open relative to R, but it is not open relative to
Rn .
Remark.
Closed relative to Y needn’t imply closed relative to X. For example, a convergent se-
quence of S that converges in X needn’t converge in Y . As a result, if this sequence that
converges in X (but not in Y ) converges outside S, under the subspace topology of Y ,
this simply does not contribute as a limit point. Whereas, in X this contributes as a limit
point, and hence is not closed in X.
Remark.
Note that, we needn’t define the concept of "relative limit point" since every limit point
relative to Y , is a limit point of S relative to X. But the back direction needn’t be true.
i.e, you can have x a limit point of S relative to X, but not relative to Y . More concretely,
x is such that for every ε > 0, there exists z ∈ S so that z ̸= x and d(z, x) < ε. If z is in
X as well as Y , its a limit point of S with respect to both. Issue arises if x is not in Y .
Then it does not make sense.
24 Metric Spaces
Theorem 1.64
A set E ⊆ Y ⊆ X is open relative to Y ⇐⇒ ∃G ⊂ X that is open relative to X, such
that E = G ∩ Y
=⇒ ) Say E is open relative to Y . This means that ∀x ∈ E, ∃εx > 0 such that if
y ∈ Bεx (x) and y ∈ Y , then y ∈ E. Call G = ∪x∈E Bεx (x) which is an open set. If
z ∈ E, then z ∈ G obviously, and hence z ∈ G ∩ Y . Hence, E ⊆ G ∩ Y . Consider a point
z ∈ G ∩ Y which means z falls in one of the ε-balls around a point of E, and z is in Y .
From definition of open relativeness, we see that z ∈ E. Hence, E = G ∩ Y
Fact 1.65
Topological definition of "open-relative": Let A ⊆ Y ⊆ X. A is said to be open relative
to Y if there exists an open set G, open in X so that A = G ∩ Y .
Theorem 1.66
A set S is open relative to Y ⊆ X if and only if Y \ S is closed relative to Y
Once we notice that replacing Bε (x) ∩ Y with BεY (x), i.e, the corresponding ε ball of x
with respect to Y , the proof falls in much the same way as the earlier version, done for
X. ■
Theorem 1.67
S is closed relative to Y ⊆ X if and only if S = H ∩ Y for a closed set H closed in X
Say S is closed, that means Y \ S = K is open relative to Y . That means there exists G
open relative to X so that G∩Y = K. Y \(K) = Y ∩K C = Y ∩(G∩Y )C = Y ∩(GC ∪Y C ) =
(Y ∩ GC ) ∩ (Y ∪ Y C ) = Y ∩ Gc . We have that Y \ K = Y \ (Y \ S) = S = Y ∩ GC .
Theorem 1.68
Suppose A1 , A2 · · · , An · · · ∈ X. Then,
2. B = ∪∞ ∞
i=1 Ai , B̄ ⊇ ∪i=1 Āi with possibility of strict inequality.
Suppose x ∈ ∪ni=1 Āi . Which means x ∈ Āi for some i. It is clear that x is either a point
of Ai or a limit point of Ai . We have that, whatever maybe the case either x is a point in
Bn or a limit point of Bn . Therfore B¯n ⊃ ∪ni=1 Āi .
Suppose x is a point in B¯n . If it is a point of Bn , we are done. Suppose it is the limit point
of Bn , but not a point. Also suppose that x is not a limit point of any Ai : i = 1 → n.
This means that,
Theorem 1.70
The Interior is an open set
SC ⊆ S¯C
Theorem 1.71
S = S ⇐⇒ S is open
=⇒ ) if S = S, obviously S is open.
Theorem 1.72
S is the largest open set contained in S
Theorem 1.73
(S)C = (S C )
"The compliment of the interior is the closure of the compliment"
Alternate method(slicker):
Theorem 1.75
Let X, dX and Y, dY be isometric under the map φ : X → Y . Then the map φ is
injective, and its inverse φ−1 : ϕ(X) → X is also also an isometry.
Theorem 1.76
Let Z be a set and f : Z → (X, d) be any injective map from Z to X. Then δ(x, y) :=
d(f (x), f (y)) would form a metric on Z and make it a metric space, and this would in
turn make f an isometry from (Z, δ) to (X, d)
δ(x, y) = d(f (x), f (y)) would obey all the properties of a metric space, and moreover,
δ(x, y) = d(f (x), f (y)) making it by definition an isometry. ■
Theorem 1.79
x ∈ A ⇐⇒ d(x, A) = 0
Remark.
In some sense, being an isolated point of a set is the opposite of being a limit point. x is
a limit point of S if for every ε > 0, there exists a point sε ∈ S \ {x} so that sε ∈ Bε \ {x}
or rather for every ε > 0, Bε (x) \ {x} ∩ S ̸= ∅. The negation of this statement is that
there exists an ε > 0 so that Bε (x) \ {x} ∩ S = ∅
Theorem 1.83
∂(S) = S \ S ◦
∂S was defined as the set of all points x so that dist(S, x) = dist(x, S C ) = 0. By virtue
of that, x ∈ ∂S implies x ∈ A. Can x ∈ S ◦ ? That would mean that there is an epsilon
ball around x ∈ S ◦ which means that the distance between x and S c would be non zero.
Hence, ∂S ⊆ S \ {S ◦ }
Fact 1.84
Boundary of a set is closed (∂(S) = S ∩ S C ).
30 Metric Spaces
Theorem 1.87
Let S ⊆ Z ⊆ X. Then,
clsZ (S) = clsX (S) ∩ Z
Note that clsX (S)∩Z is a closed set, closed relative to Z that contains S. Hence, clsZ (S) ⊆
clsX (S) ∩ Z. clsZ (S) is the smallest closed set relative to Z that contains S, which means
clsZ (S) = H ∩ Z for some closed set H. Note that this closed set must too contain S.
Hence, we have clsX (S) ⊆ H which gives clsX (S) ∩ Z ⊆ H ∩ Z = clsZ (S). Hence we have
clsZ (S) = clsX (S) ∩ Z. ■
Theorem 1.88
Let S ⊆ Y ⊆ X. Then intY (S) = intX (S ∪ (X \ Y )) ∩ Y
Theorem 1.90
A set A is dense in X if and only if for every open set G ∈ X, A ∩ G ̸= ∅
Theorem 1.91
If U is a topology arising from δ(x, y), then the same topology can also be achieved by
the metric d(x, y) = δ(x, y)/(1 + δ(x, y)), as well as e(x, y) = δ(x, y)/2
Given a topology of X, we would like to classify, or have the structure of the topology
generated in a subspace Y ⊂ X.
Theorem 1.92
If U is the topology of X, then U ∩ Y , that is {U ∩ Y : U ∈ U} is the topology of Y.
Theorem 1.93
Suppose Z is a metric space and Z ⊆ X. Topology of X includes that of Z if and only
if Z is open in X.
This essentially means that every set open relative to Z is open relative to X
if and only if Z itself is open in X.
=⇒ ) Suppose the topology of Z is contained in X, that means that every open set
relative to Z is actually an open set relative to X. That makes Z an open set relative to
X. We are done. ■
Question: Are there non empty metric spaces such that they are open relative to every
superspace?
Answer: No. Consider X to be a non empty metric space with distance d. Consider
X × {0} = Y . It is obvious that Y is bijective to X. Consider f : X → Y given by
f (x) = (x, 0). Under the obvious metric k[(x, 0), (y, 0)] = k[f (x), f (y)] = d(x, y), we can
clearly see that Y, k forms a metric space isometric to X, d. We can therefore identify X, d
with Y, k. Now look at Z = X × [0, 1] with the metric δ[(x, rx ), (y, ry )] := d(x, y) + |rx − ry |.
Consider distZ [(x0 , 0), Z \ Y ]. This is distZ [(x0 , 0), X × (0, 1]] which is 0. Hence, Y is not
open wrt Z. Its over.
inside FkC . Around this ball, though, only finite points of xn exists. This contradicts the
fact that x is a limit of (xn ). Hence, x ∈ Fk for all k ∈ N. Hence x ∈ ∩n∈N Fn . Since
diam(Fn ) → 0, its obvious that two points cannot exist in the final intersection.
⇐= ) Let (xn ) be a cauchy sequence. Note that, if {xn : n ∈ N} has a limit point,
say x, then choose ε1 = 1 and pick xk1 in this 1-ball. Then, look at the set {xn : n ≥ k1 }.
This set still has x as its limit point, wherein you choose ε2 = 1/2 and get the corre-
sponding xk2 in the 1/2−ball of x. As such keep going to get a subsequence xkj that
converges to x. We know that ∀ε > 0, ∃n0 so that ∀n, m ≥ n0 , d(xn , xm ) ≤ ε/2, more
specifically, ∀n, kj ≥ n0 , d(xn , xkj ) < ε/2. Moreover, ∀ε > 0, ∃n′ so that ∀kj ≥ n′ we
have d(xkj , x) < ε/2. Adding these two gives us that xn → x. Therefore, we assume that
{xn : n ∈ N} has no limit point. Let Fm := {xn : n ≥ m}. Each of these sets, by virtue
of having no limit points, are closed. They are, as well, nested and obviously non empty.
Moreover, diam(Fl ) := sup{d(xn , xm ) : m, n ≥ l}. If ε > 0 is given, there exists a l0 so
that ∀n, m ≥ l0 , we have d(xm , xn ) < ε which means sup{d(xm , xn ) : n, m ≥ l0 } ≤ ε.
Hence, diam(Fn ) → 0. Hence, from hypothesis, ∩n∈N Fn = {x}. d(xn , x) ≤ diam(Fn ),
which means that xn → x. Hence, cauchy complete. ■
Theorem 1.96
Cauchy completeness ⇐⇒ completeness
triangle inequality for these. Is δ(a, b) = d(a, b) ≤ δ(a, x) + δ(b, x) = limn→∞ d(a, xn ) +
limn→∞ d(b, xn )? We have the RHS limn→∞ (d(a, xn ) + d(b, xn )) which would be larger than
d(a, b). Now let a ∈ X and x = x. Let b ∈ X. We want to show δ(a, x) = limn→∞ d(a, xn ) ≤
δ(a, b) + δ(b, x) = d(a, b) + limn→∞ (b, xn ) In essence we want to show that limn→∞ d(a, xn ) ≤
limn→∞ (d(a, b) + d(b, xn )). Notice that the right hand side is always larger than d(a, xn ),
which is still preserved in the n → ∞ limit. Hence, triangle inequailty is verified. Hence, δ
is a metric.
Example : Two disjoint closed subsets X, Y of R that have d(X, Y ) = 0
Consider the sequence of irrational numbers x1 , x2 , · · · that is monotonically increasing
and divergent (to +∞). Let this be X. Consider another sequence, likewise monotonic
increasing and likewise divergent, yn of rational numbers obeying the property d(xk , yk ) <
1/k. We are done. ■
Lemma 1.97
If A is a set in a metric space X, and A is closed, then A can be written as the union
of the set of isolated points of A and the set of limit points of A (disjoint union).
Lemma 1.99
D is nowhere dense =⇒ its complement is dense. Converse needn’t be true
2 Compactness
Remark.
The notion of Being open depends largely on the metric space one is talking about. For
example, we see that certain sets may be open relative to Y ⊂ X, but not X in itself.
This is not the case for compactness though, as shall be seen.
Remark.
Note that the above theorem "compact-relativeness is conserved" did not use any property
of metric spaces, like distances or balls, so this theorem holds in any general Topological
space.
Fact 2.4
Every finite set in X is compact
Proof. Consider an open cover Gα for finite set E. This means that, for every point
x1 , x2 , · · · , xk in E, there would exist some {α1 , α2 , · · · } collection of "α-s" that is utmost
finite, such that xj ∈ Gαj . Simply take the union of Gαj to get a finite subcover.
Theorem 2.6
Closed balls in X are closed
diam(A) := sup{d(x, y) : x, y ∈ A}
It is finite if and only if it is bounded. It would be infinite if unbounded.
Lemma 2.8
If xn is a cauchy sequence and {xn } the set contains a limit point, then the cauchy
sequence converges.
Figure 1.1: Figure for the proof: Closed balls are closed
δ < min{d(x1 , x)} and get a corresponding xn2 . Then choose δ < min{xn2 , x1 } and keep
going to create a subsequence of {xn } that converges to x. ∀ε/2 > 0 ∃n′ so that ∀nk ≥ n′
we have d(xnk , x) < ε/2. Therefore, ∀ε > 0, ∃q = max n′ , n0 so that ∀n, nr ≥ q, we have
d(xn , xns ) < ε/2 and d(xns , x) < ε/2, Adding these two we get the desired result. ■
Theorem 2.9
A metric space X is complete if and only if for every sequence of nested non-empty
closed sets {Fn : n ∈ N} such that limn→∞ diam(Fn )=0, there exists one point x ∈
∩∞i=1 Fi
means it is finally in an open set. Outside any Fj , only finite points of the sequence exists.
This immediately contradicts the previous result, since x is a limit point of the sequence,
but it is in some Fjc which contains only finite points of the sequence so it is impossible
for a particular (chosen) ε−ball to contain infinite points of {xnk }. Hence, we are done.
x ∈ ∩∞ i=1 Fi . Moreover, since diam(Fn ) → 0, it is trivial to see that only one point survives
38 Metric Spaces
the intersection. (If there are two points,we can always make epsilon smaller than their
fixed distance).
⇐= ) Suppose {xn } is a cauchy sequence, i.e, ∀ε > 0 ∃n0 so that for all m, n ≥ n0 ,
d(xn , xm ) < ε. Look at Sm := {xn : n ≥ m}. If any of these sets has a limit point, then
we would be done from the previous lemma. So we assume these all dont have a limit
point. Hence they are closed, nested sets. Moreover, ∀ε > 0, ∃n0 so that ∀n, m ≥ n0 (or
rather, for any two points x and y in Sn0 ) we have d(xn , xm ) < ε(or d(x, y) < ε) which
means diam(Sn0 ) < ε. This means diam(Sn ) → 0. This means that ∩∞ i=1 Si = {x} for
some element x. x is in every Si . Let ε > 0. There exists Snε so that diam(Snε ) < ε which
means d(xnε , x) < ε which means xnε forms a convergent subsequence, which means the
sequence is finally convergent from previous lemma. ■
Theorem 2.10
Compact sets are closed.
Method 1:
Method 2:
Consider E to be compact, i.e, for every closed collection {Fα } such that ∩α Fα ⊂ E c ,
there exists a finite sub collection {Fα1 , Fα2 · · · Fαk } such that ∩kj=1 Fαj ⊂ E c . Consider a
point p outside E, i.e, in E c . Notice that ∩ε∈R+ B[ε] (p) = {p} which is in E c . This would
be a collection of closed sets whose intersection falls completely inside E c . Hence, there
would exist a finite subcollection such that ∩kj=1 B[εj ] (p) ⊂ E c which means there would
exist a neighbourhood around p which is completely in E c . Hence, E c is open, and E is
closed.
■
Fact 2.11
ϕ and X are both open and closed.
Metric Spaces 39
Theorem 2.12
Closed subsets of compact sets are compact
Corollary 2.13
If F is closed, and K is compact, then F ∩ K is compact
Fact 2.14
A compact set is bounded
Proof. Consider (WLOG, a non empty compact set E) and an arbitrary point q in X. Bε (x)
for every ε > 0 forms an open cover for E (since it is basically X). Which means there is a
finite subcover, i.e, a number ε0 > 0 such that E ⊂ Bε0 (p) which makes E bounded.
Theorem 2.15
Finite union of compact sets is compact
Theorem 2.16
If {Kα } is a collection of compact sets such that for every finite subcollection
{Kαj : 1 ≤ j ≤ k} we have that ∩kj=1 Kαj ̸= ϕ. Then ∩α Kα ̸= ϕ. In pithy words:
"If you have a collection of compact sets for which every finite subcollection’s
intersection is non-empty, the intersection of the whole collection is non empty"
-Krishna, to Arjuna
Suppose, on the contrary, let ∩α Kα = ϕ which means ∪α Kαc = X which means for every
for some α0 , we have Kα0 ⊂ ∪α Kαc , where ∪α Kαc is an open cover of Kα0 . This implies
that there exists a finite subcollection {KαC1 , KαC2 · · · KαCr } such that Kα0 ⊂ ∪rj=1 KαCj =⇒
∩rj=1 Kαj ⊂ KαC0 . But this means ∩rj=1 Kαj ∩ Kα0 = ϕ, which is absurd since all finite
intersection is non empty.
■
Corollary 2.17
If K1 , K2 , · · · is a sequence of non-empty compact sets such that · · · Kn ⊂
Kn−1 · · · K3 ⊂ K2 ⊂ K1 , then ∩∞i=1 Ki is non empty.
Suppose that E has no limit point in K. Since K is closed, E must have no limit points.
Hence, E is closed. Since closed subsets of compact sets are compact, E is compact. If no
point of E is a limit point of E, then ∀x ∈ E, ∃εx > 0 such that no point of E apart form
x itself falls into the εx -ball of x. Consider the open cover {Bεx (x) : x ∈ E} of E. This has
a finite subcover {Bεx1 (x1 ), Bεx2 (x2 ), · · · Bεxl (xl )}. We see that E ⊆ ∪lj=1 Bεxj (xj ). But
since for every εxj -ball around xj , no point in E except xj resides, ∪lj=1 Bεxj (xj ) will have
utmost finite points. Since an infinite set E cannot be the subset of a finite set, we have
a contradiction. ■
Theorem 2.20
k-cells are closed
Consider a k-cell E. Consider a point z not in E, i.e, ∃j0 such that either zj < aj or
zj > bj . WLOG, take the case of zj < p aj . Let 0 < δ < (aj − zj ). Consider a point q in the
δ-ball around z. i.e, d(z, q) < δ =⇒ (z1 − q1 )2 + (z2 − q2 )2 + · · · + (zk − qk )2 < δ =⇒
(z1 − q1 )2 + (z2 − q2 )2 + · · · + (zk − qk )2 < δ 2 < (aj − zj )2 =⇒ 0 < (qj − zj )2 < (aj − zj )2
=⇒ qj < aj . Hence q ̸∈ E, which implies there exists, for every x in E c , a δ for which the
δ-ball around x is fully contained in E c which means E c is open. This implies E is closed.
Same argument applies for the case where zj > bj . ■
Theorem 2.21
Closed intervals in R are compact
Let I be, WLOG, [−a, a]. Suppose it is not compact. i.e, There is an open cover Gα of I
such that there exists no finite subcover. ∀x ∈ I, ∃αx such that x ∈ Gαx and ∃εx such that
Bεx (x) ⊂ Gαx . ∪x Bεx (x) ⊂ ∪α Gα is an open cover for I. note that, if no finite subcover
for Gα exists, then no finite subcover for Bεx (x) exists either. So we can safely work with
Bεx (x). Split the interval into two halves, [−a, 0] and [0, a]. One of these intervals is not
finitely covered by Bεx (x), for if not, the whole thing would be finitely covered. let that
interval which is not finitely covered be I1 . This interval’s size is a. Split this interval
into two again. Yet again, one of the halves must not be finitely covered, for if not, I1
would be finitely covered, which is contradictory. Let this interval be I2 . This is of size
a
2
. Yet again, keep doing this process to obtain a sequence of intervals Ij , sized aj , which
are not finitely covered. These are nested intervals, non empty, and closed. From nested
intervals theorem, we see that a point ξ exists in ∩∞ j=1 Ij . ξ is a point in I, and there is a
a εξ
corresponding εξ . Consider that j0 for which j0 < 2 . We know from Archimedean such a
j0 exists. This means that the interval Ij0 containing ξ, sized ja0 , is completely inside the
εξ -ball around ξ, which means it is finitely covered. Contradiction. Hence, I is compact.
■
Corollary 2.22
Since intervals of the form [−a, a] are compact, every closed interval of the form [a, b]
is compact since it would be a closed subset of an interval of the form [−x, x].
Generalisation:
42 Metric Spaces
Theorem 2.23
n-cells are compact
Remark.
We proved the result for k-cells of the kind [−a, a]k , but it is easily generalised by noting
that arbitrary k-cells are contained in some k-cell of the above kind. By virtue of being
closed, they also are compact.
2. E is compact
Figure 1.2: Figure for the proof: n-cells are compact.(The εp -ball around p, and the n-cell
construction)
Theorem 2.25
If {xn } is a sequence in X convergent to x ∈ X, then the set {xn } has only one limit
point, which is x.
That x is a limit point is clear. We note that ∀ε > 0, ∃n0 such that ∀n ∈ N, n ≥ n0 we
have d(xn , x) < ε. i.e, beyond a particular n0 , every point of {Xn } falls in the ε-ball of
x. Therefore, only finite points lie outside this ε-ball of x. Suppose it has another limit
point y, other than x. Therefore, there would exist a δ such that the δ-ball around y lies
completely outside the δ-ball around x. This means that, only finite points of xn lie in the
δ ball of y, making it unviable to be a limit point. ■
Extending Heine Borel we have:
44 Metric Spaces
2. E is compact
(3) =⇒ (1)) Let us assume that E is either not closed, or not bounded. We start
by assuming it is not closed. Which means that ∃q outside E such that there exists a
sequence in E that converges to q. We take this sequence {xn } as our infinite set, and we
see that, from the previous theorem, this has only one limit point q, which lies outside E.
Hence, there exists an infinite set {xn } which has no limit point in E.
Remark.
In the previous proof, we note that (3), which is called Limit Point Compactness, implies
(1) Closed and Bounded, in any metric space, not just Rn , as we see in the proof, no
property of Rn was used.
Figure 1.3: Figure for proof: Lim point compact =⇒ closed+bounded. (The construction
of an unbounded sequence)
Remark.
The above "Weierstrass Theorem" is just the "Bolzano-Weierstrass" Theorem we saw in
sequences. Actually, the "Bolzano-Weierstrass" Theorem is a direct corollary of the more
general "Weierstrass Theorem". Let {xn } be any sequence in R that is bounded. This
means that this sequence is the subset of a compact set, hence, has a limit point in R.
This implies, a subsequence of {xn } converges in R. Hence, every bounded sequence has
a convergent subsequence.
Fact 2.28
Let X = Rn . The closure of any open ball is the corresponding closed ball.
Proof. Consider B := Bδ (x0 ) := {y ∈ Rn : ||y − x0 || < δ}. Let z0 be a point on the rim
of B, i.e d(x0 , z0 ) = δ. Such a point obviously exists. Consider ⃗γ (t) = t⃗z0 + (1 − t)⃗x0 with
46 Metric Spaces
t ∈ (0, 1). For every t ∈ (0, 1), ⃗γ (t) belongs in B. To see this, consider ||⃗γ (t) − ⃗x0 || =
||t⃗z0 + (1 − t)⃗x0 − ⃗x0 || = ||t(⃗z0 − ⃗x0 )|| = t||⃗z0 − ⃗x0 || < t(δ) < δ. Suppose we are given
an arbitrary η > 0. Does there exist a t ∈ (0, 1) so that ⃗γ (t) belongs in the η-ball of ⃗z0 ?
i.e, we need a t so that ||⃗γ (t) − ⃗z0 || = ||t⃗z0 + (1 − t)⃗x0 − ⃗z0 || = ||(1 − t)(⃗z0 − ⃗x0 )|| < η
=⇒ (1 − t)||⃗z0 − ⃗x0 || < η =⇒ 1 − t < ηδ =⇒ 1 − ηδ < t < 1. Such a t exists for
every η. Hence, ⃗z0 is a limit point of B (by virtue of there existing a sequence of ⃗γ (tj ) that
converges to ⃗z0 ). Hence, every point on the rim is a limit point. Moreover, no point w so
that d(w, x0 ) > δ is a limit point of B, since there would exist an ε-ball around w so that no
point of B falls into it (from openness). Hence, closure of B is the corresponding closed ball,
in Rn .
Theorem 2.30
A is dense in X if and only if A = X if and only if for every open set U of X, A ∩ U ̸= ∅
3 Perfect Sets
Theorem 3.2
Perfect subsets in Rn are uncountable.
Choose x1 , and ε0 = 1. Let V0 denote the ε0 -ball around x1 . This ball is non empty,
Metric Spaces 47
moreover, V¯0 ∩ E(which is the corresponding closed ball of V0 ) is non empty, and is com-
pact by virtue of being closed and bounded. Inside, V0 ∩ E, there exists infinite points of
E, since x1 is a limit point of E.
Choose an arbitrary point z1 in V0 that is not x1 . Now let ε1 < d(x1 , z1 ). Let V1 be
the ε1 -ball around z1 . Notice the following: z1 is a limit point of E, hence, there are
infinite points of E in V1 . x1 is not in V¯1 . V¯1 ∩ E is closed, bounded and non empty, hence
Compact.
Choose a point z2 in V1 that is not x2 , and let ε2 < min{ε1 , d(x2 , z2 )}. Let V2 be the
ε2 -ball around z2 . Note that, x2 is not in V¯2 . Also note yet again that there are infinitely
many points of E in V2 . It is crucial to note now that V¯2 ∩ E ⊂ V¯1 ∩ E ⊂ V¯0 ∩ E.
Suppose you have already constructed Vk by finding zk in Vk−1 that is not xk and an
εk < mind(zk , xk ), εk−1 such that xk ̸∈ V¯k , V¯k ∩ E is compact, non empty and V¯k ∩ E ⊂
¯ ∩ E ···.
Vk−1
Now, choose zk+1 ̸= xk+1 , inside Vk . Choose εk+1 < min{d(zk+1 , xk+1 ), εk }. Let Vk+1
¯ ∩ E is non empty, xk+1 is not in
be the εk+1 -ball around zk+1 . Yet again, we see that Vk+1
¯ , and Vk+1
Vk+1 ¯ ∩ E ⊂ V¯k ∩ E. Hence, we have a sequence of non empty, nested compact
sets. This implies that ∃ξ ∈ E ⊂ Rn such that ξ ∈ ∩∞ i=1 (V̄i ∩ E). Is ξ any one of xj
enumerated? No, because if it was, from the construction, xj would not belong in Vj .
Hence, ξ is not in the enumeration of E. Contradiction. ■
48 Metric Spaces
Figure 1.4: Figure: Perfect sets are uncountable. Construction of the nested sequence of
compact sets by choosing zk ̸= xk ∈ Vk−1 .
Remark.
It is easily seen that, closed intervals in R are perfect: From density theorem, for every
point in I, there would exist a sequence of rationals converging to that point. Moreover,
closed intervals in R are closed since closed balls in metric spaces are closed. Therefore,
we see that intervals are uncountable.
Let I0 = [0, 1]. size of the interval(s) in I0 is 1, and there are 20 = 1 intervals.
Let I1 = [0, 31 ] ∪ [ 23 , 1] be constructed by trisecting I0 and tossing the middle one. Here,
we have each interval sized 311 , and there are 21 = 2 intervals total.
vals in I1 , trisecting them, and tossing the middle one, and joining them finally. We have
each interval sized 312 and there are 22 = 4 intervals total.
Note that P is compact since it is the closed subset of a compact set. It is also non empty
by virtue of being the intersection of a sequence of nested, non empty, compact sets.
Note that, no interval of the kind [a, b] exists in the Cantor Set. The size of each inter-
val in Ij is 31j . We can find j so that 31j < b − a =⇒ b−a 1
< 3j =⇒ log3 ( b−a 1
) < j. For
such Ij , we notice that [a, b] has "inbetween" points that doesn’t exist in any of Ij ’s intervals.
Hence, taking the intersection, these "inbetween" terms don’t survive. Hence, no intervals
exist.
Theorem 3.3
The Cantor set P is perfect.
We already know that the Cantor set is closed. We need to show that every point in the
cantor set is a limit point. First, observe that, for any Ik , if z is the end point of any of
the sub interval of Ik , it survives the ∞-intersection. This is because, after Ik -s trisection,
the end points still stay endpoints. Let ξ be any point in the cantor set, which means
it is a point in every Ik . Let δ > 0 be given. Consider the interval (ξ − δ, ξ + δ). This
interval is sized 2δ. ξ exists in one of the sub intervals of Ik for all K ≥ k0 for some k0 .
Choose j so that 31j < δ. Then, the interval in Ij containing ξ would fall completely inside
(ξ − δ, ξ + δ). Choose q as one of the end points of this sub interval of Ij . Therefore,
∀ξ ∈ P , ∀δ > 0, ∃q ∈ P, q ̸= ξ so that q ∈ (ξ − δ, ξ + δ). Therefore, every ξ ∈ P is a limit
point of P . Hence, P is perfect. ■
4 Connected Sets
Theorem 4.3
E ⊂ R is connected ⇐⇒ ∀x, y ∈ E, x < z < y =⇒ z ∈ E.
⇐= ) Suppose that we have E disconnected, which means it is the union of two separated
sets A and B that are non-empty. x0 ∈ A and y0 ∈ B. Consider z(t) = x0 + t(y0 − x0 ) for
t ∈ [0, 1]. Note that z(0) = x0 and z(1) = y0 .
Conjecture: There exists a tB ∈ (0, 1) so that for every t < tB , z(t) does not belong
in B. If it is not true, then for every t ∈ (0, 1), there exists a point tB < t so that z(tB )
is in B. Choose t = 1 to get z(t1 ) in B. Chooe t = t21 to get z(t2 ) in B with t2 < t1 and
t2 < 12 . Keep going with t = 2tn−1 1
n−1 to get z(tn ) in B with tn < tn−1 and tn < 2n−1 . This
gives us a sequence z(tk ) which we can see is monotone decreasing assuming x0 < y0 . This
sequence converges to z(0) which is in A which means that there exists a sequence in B,
z(tn ) that converges to A. Absurd.
In a similar vein, we can show that there exists tA ∈ (0, 1) so that for every t > tA ,
z(t) is not in A. Consider
and
SB := {t ∈ [0, 1] : z(t) ∈ B ∩ [x0 , y0 ]}
It is easy to see that SA and SB are disjoint. If a sequence in one converges in another,
say tn ∈ SB converges to t0 ∈ SA . Then z(tn ) ∈ B by definition, for every n. But then
by definition, z(tn ) = x0 + tn (y0 − x0 ) ∈ B such that lim(z(tn )) = x0 + t0 (y0 − x0 ) ∈ A,
which means a sequence in B converges in A. Absurd. So SA and SB are separated.
Metric Spaces 51
Note that, for t > tA , no z(t) is in A. Hence, we see that for every t so that z(t)
falls in A, there is an upperbound. Likewise, for every t such that z(t) falls in B, there is
a lowerbound. Hence, SA has a supremum sup(SA ) and SB has an infimum inf (SB ).
At this point, we may as well assume that for every t < inf (SB ), t ∈ SA for if not,
what we wanted to prove would get proved. Suppose then, for argument sake, that for
every t > Sup(SA ), t ∈ SB , and likewise, for every t < Inf (SB ). t ∈ SA . Now then, does
Sup(SA ) belong in SA ? we see that for every t > sup(SA ), t ∈ SB which means we can
construct a sequence in SB using those ts, which converge to Sup(SA ) in SA . So that is
ruled out. So is Sup(SA ) in SB ? That is not possible either, since SA is a bounded, infinite
set (mainly because supremum isn’t in the set), we know that there is a monotone sub-
sequence in SA converging to Sup(SA ) which is in SB . We therefore conclude that, there
exists a point t ∈ (0, 1) so that t is neither in SA , nor in SB . This translates to there being
a point z = z(t), between x0 and y0 so that z(t) ̸∈ A∪B =⇒ ̸∈ E. We are, therefore, done.
Figure 1.5: Figure: Proof for the equivalence for connectedness for sets in R. A look at
A ∩ [x0 , y0 ] and B ∩ [x0 , y0 ].
5 Misc Knowledge
Theorem 5.1
1. If A and B are closed, disjoint subsets of X, then A and B are separated.
(1) A B closed implies A = A and B = B which are disjoint. From here it is obvious.
(2) A and B are open disjoint sets, then we see that A ⊆ B C and B ⊆ AC where AC and
B C are closed by definition. Since closure is the smallest closed set containing A (and B),
we see that A ⊆ B C and B ⊆ AC . It is now trivial to see that A∩B ⊆ B C ∩B = ϕ = B ∩A
which is the definition of separated. ■
Corollary 5.2
Let p ∈ X and δ > 0. Define A := Bδ (p) and B = (B[δ] (p))C . A and B are, then,
separeted.
Easy to see that they are both open sets that are disjoint. ■
Theorem 5.3
Every connected metric space with atleast two points is uncountable.
Let a and b be in X. Let ξ ≤ d(a, b). Note that, P = Bξ (a) and Q = (B[ξ] (a))C are non
empty, separated sets (from the previous corollary). If X is not the union of P and Q,
then there is a point zξ in X so that it is neither in P not in Q. That means that it is
exactly ξ distance away from p. For every ξ < d(a, b), there exists a point zξ so that its
distance from p is exactly ξ. Therefore, every zξ is unique (from positivity property of
metric spaces) which means there are uncountable zξ -s. ■
Theorem 5.4
If P and Q are connected such that P ∩ Q ̸= ϕ, then P ∪ Q is also connected.
Lemma 5.5
Given two balls B1 and B2 in Rn that are closed, with B1 ∩ B2 = {z} with z ∈ Rn ,
then the interior of B1 ∪ B2 , i.e, B1 ∪ B2 , is B1 ∪ B2 , which are their respective open
ball counterparts.
Corollary 5.6
If A ⊂ X is connected, it needn’t be true that A is connected.
Theorem 5.7
Let E be the set of all x ∈ [0, 1] ⊆ R so that the decimal expansion of x only contains
4 and 7. Then:
1. E is uncountable
3. E is compact
4. E is prefect
(3) We already know E is bounded. Consider E c . This is the set of all numbers in
[0, 1] so that not all points in the decimal expansion is 4 or 7. i.e, there would be a point
in the expansion that is neither 4, nor 7. Suppose we take one such arbitrary x ∈ E c . Let
the first non 4, 7 number occur at the j−th place. 0.z1 z2 z3 · · · xj · · · . Look for another
non 4, 7 after the j−th place (if it exists). If it doesn’t exist, then all the numbers after xj
54 Metric Spaces
would be 4 or 7 so safely add 10−(j+1) as our ε. This ε range around x would contain only
points of E c . Suppose another point exists that is non 4, 7 after j, perhaps at k > j-th
index. Then it would look something like: 0.z1 z2 · · · zj xj+1 xj+2 · · · zk · · · . Here we simply
take ε = 10−(k+1) so that all points in the ε-neighbourhood of x is in E c . Therefore, E c is
open, which means E is closed. Closed and bounded implies compact in R.
We saw that E is closed. We need only show that every point of E is a limit point
of E. This can be done easily for any ε-ball, using the technique that follows: Choose a
k so that 101k < ε. Look at the interval x − 101k , x + 101k that is contained in E. Just find
some n > k, and flip the 4 to a 7 or vice versa to land in a "different" element from x, yet
within the neighbourhood in consideration. Hence, every point is a limit point, making E
a perfect set.
■
point would be q. Hence, q = 0. This means that the only limit points of Φ other than
1
j
is 0. Hence, we have a countable limit point. Hence, Φ is a closed set and bounded
obviously, with countable limit points. ■
SA := {t ∈ R : p(t) ∈ A}
SB := {t ∈ R : p(t) ∈ B}
Then:
(2) Since SA and SB are separated and non-empty, there are two points x0 and y0 in
SA and SB respectively. Define z(l) = x0 + l(y0 − x0 ) for l ∈ [0, 1]. Now, for some lA , we
have that for every l > lA , z(l) ̸∈ SA , the set GA := {l : z(l) ∈ SA } is therefore bounded
above with supremum uA . Likewise for some lB , we have that for every l < lB , z(l) ̸∈ SB ,
the set GB := {l : z(l) ∈ SB } is therefore bounded below with infimum vB . Note that GA
and GB are separated sets. We may as well assume that for every l < lB , l is in GA , or
z(l) falls in SA . If not, we would be done. We now ask: does vB fall in GA or GB ? If
it falls in GB , there exists a sequence in GA that would converge to vB , which is absurd.
If it falls in GA , then by virtue of being the infimum of GB , there is a sequence in GB
converging in GA . Hence, there exists a point l between x0 and y0 l ̸∈ GA or GB which
means z(l) ̸∈ SA or SB . This again means that p(z(l)) ̸∈ A or B. Phew. ■
Corollary 5.10
Every convex set in Rn is connected.
2. E is non compact.
One way to see that E is non compact is simply by making use of the "conservation"
of compactness going from one space to a bigger space or vice-versa. Since E is clearly
not compact in R, it wont be compact in the metric subspace Q. Another way to see
that it is non compact√is to√consider the√ following
√ construction:
√ √ Look at the union of the
two split intervals (− 3, − 2) and ( 2, 3). Let h = 3 − 2. We construct √ it for the
right side
√ interval, and simply copy it to the left one. Choose the point 3 and a h/2-ball
around
√ 3 and call it V0 . This would intersect the right interval at a distance h/2 from
3. Choose this intersection point and a h/4-ball around this called V2 . Both V1 and V2
together covers 3h/4 of the interval. Choose this intersection point and let the h/8-ball
around this point be V3 . V1 , V2 and V3 together cover 7h/8 of the interval. Keep going as
such to construct Vn so that (Vi )ni=1 covers (n−1)h
n
of the whole interval. As n tends to ∞,
the "coverage" converges to h. This means that for every ε distance away, there exists a
finite n0 so that V1 → Vn0 covers up to that ε distance. Every point e in the strict interval
would therefore be covered up by some Vk by our construction. But obviously, this "open
cover" has no finite subcover, for no finite "coverage" covers all the way till h distance of
the interval. Some ε-gap is always left, hence missing points.
√ √
E can also be written as the√disjoint union
√ of the set A of all p so that 2 <
√ p < 3√
and
so that − √
the set B of all p √ 3 < p < − 2. WLOG say q ∈ A. Obviously 2 < q < 3.
Choose δ < min{ 3 − q, q − 2} and the δ−ball called V around q. Easy to see that this
ball V is fully contained in A. Likewise, it can be shown for B as well. Hence, E is open
with respect to Q.
■
Example : Rn is separable
Consider the set of all points z ∈ Rn with coordinates in Q. Basically Qn . This would be
a countable set, and every point x ∈ Rn is a limit point of this set (since coordinate we
can have a rational sequence converging to that coordinate) ■
Theorem 5.14
For a metric space X, separability ⇐⇒ countable basis
1
n
< δ. In this 1/n ball around z, there would exist a point xk in the dense set. Choose
now, the 1/n ball around xk which contains z, and would be completely contained in the
εG
z ball, which would be contained in G. Hence, we are done.
⇐= ) Say X has a countable basis {V1 , V2 , · · · } that are non empty. Choose x1 ∈ V1 ,
x2 ∈ V2 · · · . We claim that this set {x1 , x2 · · · } forms our countable dense set. Say a point
z ∈ X, choose any arbitrary ε > 0. The ε−ball around z would be an open set, which
means a set Vk is inside ε−ball around z. This would mean that xk would be in the set,
which makes z a limit point of this supposed to be dense set {x1 , x2 · · · }. We are done.
■
58 Metric Spaces
Theorem 5.15
⇐⇒
∃{Vα : α ∈ A}(∀G ⊂ X : G open in X)(∃A′ ⊆ A)(G = ∪α Vα : α ∈ A′ )
Or in pithy words,
Vα is basis if and only if every open set is the union of a subcollection of {Vα }
Fact 5.16
Definition 5.17
2nd countable
Theorem 5.18
Let X be a metric space in which every infinite subset E has a limit point in X. Then
X has countable basis (or equivalently is separable).
Note that no infinite subset of X can be "unbounded" since we have seen before that Limit
point compact implies closed and bounded. Consider an arbitrary δ0 . Choose an initial
point x1 . Is there a point x2 that is outside the δ−ball around x1 ? If no, the only δ−ball
of x1 covers the whole space. If yes, then again ask the question, is there a point x3 that
is both outside the δ−ball of x1 and the δ−ball of x2 ? If not, then these two balls will
cover the whole space, if yes, again ask the question, is there a point x3 so that it is not
in x1 , x2 and x3 ’s δ−balls. Keep going, as such. We claim that it must terminate after a
finite number of steps. Suppose not, i.e for every xn you can find, you can find an xn+1 to
form an infinite set of xj such that xj is not in the δ-ball of any of its preceeding elements
xj−1 , xj−2 · · · . This is true for every xj . From the hypothesis, this set has a limit point
q. Choose ε < δ/4, within which exists a point xk in this infinite set. But since no point
exists within the δ−ball of xk apart from itself, no other point exists in the ε−ball around
xk as well. This would contradict the proposition that q is a limit point. Hence, this
procedure must terminate in a finite amount of steps. So for a given δ = d, there exists
nδ balls V1 , V2 · · · Vnd with centres xd1 , xd2 · · · xdnd . Choose δ = 1, and create a collection of
1-balls (by the procedure mentioned above) around the points x11 , x12 · · · x1n1 . Likewise, for
δ = 1/2, find points x12 , x22 · · · x2n2 , and for δ = 1/k, find points xk2 , xk2 · · · xknk . Let z be a
point in X. Choose a ε ball around z. Let 1/n < ε. There must be some xnj so that z is
in the 1/n-ball of xnj . Hence, {xkj : j ∈ N, k ∈ N} is the dense set we need. ■
Theorem 5.19
Separable ⇐⇒ countable basis ⇐⇒ every open cover of X has a countable subcover
Theorem 5.20
A compact metric space has a countable base (or equivalently, is separable- has a
countable dense set in it).
That this space is separable is obvious now. Choose xij : i, j ∈ N . Let z be a point
in X. Choose any arbitrary ε. Find an n so that n1 < ε. From the result we have, we can
always find a xkj in our set so that it is in the n1 ball of z. This means that in every ε ball
of z, there exists a point from our stipulated set. Hence, our set is dense in X. ■
Theorem 5.21
If X is a metric space so that every infinite set in X has a limit point in X, then every
open cover of X (open relative to X) has a finite subcover. Hence:
"If X is a limit point compact metric space, then X is a compact metric space
(compact relative to itself, but it also applies to all spaces it lives in, due to
preservation of compactness)"
-Krishna, to Arjuna, at Kurukshetra
Let this countable subcover be G1 , G2 · · · Gn · · · . Suppose to this, there does not exist
a finite subcover. i.e,
∃x1 ∈ GC 1
,
∃x2 ∈ (G1 ∪ G2 )C = C1c ∩ GC
2
.
..
.
Metric Spaces 61
, for every n ∈ N. Collect all such xn s to form an infinite set in X. By hypothesis, this has
a limit point, call it z. Note that, outside a given GC k , only finite points of our stipulated
set exists, which are possibly x1 , x2 · · · xn−1 . Suppose there exists a GC C
j so that z ̸∈ Gj .
This means that z is in Gj which is an open set. Therefore, there exists an ε ball that is
completely inside Gj , or rather completely outside GC j . This means that only finitely many
x1 , x2 · · · make into this ε-ball of z which is absurd since z is supposedly a limit point.
Hence, we cannot have a countable cover that has no finite subcover. Hence, Gj : j ∈ N
has a finite subcover, which means X is a compact metric space. ■
Remark.
We showed that every limit point compact metric space is compact, i.e, every open cover,
open relative to X, has a finite subcover. Suppose X is actually a subset of a bigger set
H and X inherits the metric from H. From conservation of compact relativeness, we see
that X must be compact relative to H as well. Hence, every limit point compact set in X
is compact in X.
6. X does not have a continuous onto function mapping X to {−1, 1} with discrete
topology
1 =⇒ 5) Suppose there exists a non empty proper subset of X, call it W that has
an empty boundary. i.e, W \ (W 0 ) = ∅ which means W ∩ (W 0 )C = ∅. W C ⊆ (W 0 )C which
means W ∪ (W o )C = X which makes X the disjoint union of two closed sets