Continuous
Continuous
1 Continuous functions
Definition 1. Let (X, dX ) and (Y, dY ) be metric spaces. A function f :
X → Y is continuous at a ∈ X if for every > 0 there exists δ > 0 such that
dX (x, a) < δ implies that dY (f (x), f (a)) < .
In terms of open balls, the definition says that f (Bδ (a)) ⊂ B (f (a)). In
future, X, Y will denote metric spaces, and we will not distinguish explicitly
between the metrics on different spaces.
Definition 2. A subset U ⊂ X is a neighborhood of a point a ∈ X if
B (a) ⊂ U for some > 0.
A set is open if and only if it is a neighborhood of every point in the
set, and U is a neighborhood of x if and only if U ⊃ G where G is an open
neighborhood of x. Note that slightly different definitions of a neighborhood
are in use; some definitions require that a neighborhood is an open set, which
we do not assume.
Proposition 3. A function f : X → Y is continuous at a ∈ X if and only
if for every neighborhood V ⊂ Y of f (a) the inverse image f −1 (V ) ⊂ X is a
neighborhood of a.
Proof. Suppose that the condition holds. If > 0, then V = B (f (a))
is a neighborhood of f (a), so U = f −1 (V ) is a neighborhood of a. Then
Bδ (a) ⊂ U for some δ > 0, which implies that f (Bδ (a)) ⊂ B (f (a)), so f is
continuous at a.
Conversely, if f is continuous at a and V is a neighborhood of f (a),
then B (f (a)) ⊂ V for some > 0. By continuity, there exists δ > 0 such
that f (Bδ (a)) ⊂ B (f (a)), so Bδ (a) ⊂ f −1 (V ), meaning that f −1 (V ) is a
neighborhood of a.
1
Definition 4. A function f : X → Y is sequentially continuous at a ∈ X if
xn → a in X implies that f (xn ) → f (a) in Y .
Proof. Suppose that the inverse image under f of every open set is open. If
x ∈ X and V ⊂ Y is a neighborhood of f (x), then V ⊃ W where W is an
open neighborhood of f (x). Then f −1 (W ) is an open neighborhood of x and
f −1 (W ) ⊂ f −1 (V ), so f −1 (V ) is a neighborhood of x, which shows that f is
continuous.
Conversely, suppose that f : X → Y is continuous and V ⊂ Y is open. If
x ∈ f −1 (V ), then V is an open neighborhood of f (x), so the continuity of f
implies that f −1 (V ) is a neighborhood of x. It follows that f −1 (V ) is open
since it is a neighborhood of every point in the set.
2
Proof. Suppose that f : X → Y is continuous and X is compact. If {Gα :
α ∈ I} is an open cover of f (X), then {f −1 (Gα ) : α ∈ I} is an open cover of
X, since the inverse image of an open set is open. Since X is compact, it has
a finite subcover {f −1 (Gαi ) : i = 1, 2, . . . , n}. Then {Gαi : i = 1, 2, . . . , n} is
a finite subcover of f (X), which proves that f (X) is compact.
2 Uniform convergence
A subset A ⊂ X is bounded if A ⊂ BR (x) for some (and therefore every)
x ∈ X and some R > 0. Equivalently, A is bounded if
It follows that
3
Proof. Let a ∈ X. Since (fn ) converges uniformly to f , given > 0, there
exists n ∈ N such that
d (fn (x), f (x)) < for all x ∈ X,
3
and since fn is continuous at a, there exists δ > 0 such that
d (fn (x), fn (a)) < if d(x, a) < δ.
3
If d(x, a) < δ, then it follows that
d (f (x), f (a)) ≤ d (f (x), fn (x)) + d (fn (x), fn (a)) + d (fn (a), f (a)) < ,
Proof. The uniform Cauchy condition implies that the sequence (fn (x)) is
Cauchy in Y for every x ∈ X. Since Y is complete, fn (x) → f (x) as n → ∞
for some f (x) ∈ Y .
Given > 0, choose N ∈ N such that for all m, n > N we have
4
3 Function spaces
Definition 16. The metric space (B(X, Y ), d∞ ) is the space of bounded
functions f : X → Y equipped with the uniform metric
6
For simplicity, we now specialize to real-valued functions. In that case,
we write C(X) = C(X, R). If X is compact, then C(X) equipped with
the sup-norm kf k∞ = supx∈X |f (x)|, and the usual pointwise definitions of
vector addition and scalar multiplication, is a Banach space.
7
Since X is compact, it has a finite δ-net E = {xi : 1 ≤ i ≤ n} such that
n
[
X= Bδ (xi ).
i=1
Let f, g ∈ Fφ . Then for each xi ∈ E, we have f (xi ), g(xi ) ∈ B/6 (yj ) for
some yj ∈ F , so
|f (xi ) − g(xi )| < .
3
Furthermore, if x ∈ X, then x ∈ Bδ (xi ) for some xi ∈ E, so d(x, xi ) < δ, and
the uniform equicontinuity of F implies that
is totally bounded.
8
Conversely, suppose that F ⊂ C(X) is precompact. Then F is bounded,
so there exists M > 0 such that kf k∞ ≤ M for all f ∈ F, which implies that
F is pointwise (and, in fact, uniformly) bounded.
Moreover, F is totally bounded, so given > 0, there exists a finite (/3)-
net E = {fi : 1 ≤ i ≤ n} for F. Each fi : X → R is uniformly continuous, so
there exists δi > 0 such that d(x, y) < δi implies that |fi (x) − fi (y)| < /3.
Let δ = min{δi : 1 ≤ i ≤ n}. If f ∈ F, then kf − fi k∞ < /3 for some
fi ∈ E, so d(x, y) < δ implies that
|f (x) − f (y)| ≤ |f (x) − fi (x)| + |fi (x) − fi (y)| + |fi (y) − f (y)| < ,
un+1 = un + hf (un , tn ) .
9
Define uh (t) by linear interpolation between un and un+1 , meaning that
(t − tn )
uh (t) = un + (un+1 − un ) for tn ≤ t ≤ tn+1 .
h
Choose L, T1 > 0, and let
R1 = (x, t) ∈ R2 : |x − u0 | ≤ L and 0 ≤ t ≤ T1 .
and define R ⊂ R1 by
R = (x, t) ∈ R2 : |x − u0 | ≤ L and 0 ≤ t ≤ T .
10
tn ≤ t ≤ tn+1 . Then
n−1
X
|uh (t) − uh (s)| ≤ |uh (t) − uh (tn )| + |uh (tk+1 ) − uh (tk )|
k=m+1
+ (tm+1 − s) |f (um , tm )|
≤ M [(t − tn ) + (tn − tm+1 ) + (tm+1 − s)]
≤ M |t − s|.
Let χ[0,t] be the characteristic function of the interval [0, t], defined by
(
1 if 0 ≤ s ≤ t
χ[0,t] (s) =
0 if s > t
|x − y| < M δ and |s − t| < δ implies that |f (x, s) − f (y, t)| < /T .
11
For 0 < h < δ and tk ≤ s ≤ tk+1 , we have |uh (s) − uh (tk )| < M δ and
|s − tk | < δ, so for 0 ≤ t ≤ T we get that
Z t
uh (t) − u0 − f (uh (s), s) ds
0
N −1
X k+1Z t
≤ χ[0,t] (s) |f ((uh (s), s) − f (uh (tk ), tk )| ds
k=0 tk
N −1 Z tk+1
X
< χ[0,t] (s) ds
T k=0 tk
< .
Thus,
Z t
uh (t) − u0 − f (uh (s), s) ds → 0 uniformly on [0, T ] as h → 0.
0
for each t ∈ [0, T ]. Hence, since the limits must be the same,
Z t
u(t) = u0 + f (u(s), s) ds,
0
12
Definition 32. A family of functions A ⊂ C(X) is an algebra if it is a linear
subspace of C(X) and f, g ∈ A implies that f g ∈ A.
Here, f g is the usual pointwise product, (f g)(x) = f (x)g(x).
Definition 33. A family of functions F ⊂ C(X) separates points if for every
pair of distinct points x, y ∈ X there exists f ∈ F such that f (x) 6= f (y).
A constant function f : X → R is a function such that f (x) = c for all
x ∈ X and some c ∈ R.
Theorem 34 (Stone-Weierstrass). Let X be a compact metric space. If
A ⊂ C(X) is an algebra that separates points and contains the constant
functions, then A is dense in (C(X), k · k∞ ).
Proof. Suppose that f ∈ C(X) and let > 0. By Lemma 35, for every
pair of points y, z ∈ X, there exists gyz ∈ A such that gyz (y) = f (y) and
gyz (z) = f (z).
First, fix y ∈ X. Since f − gyz is continuous and (f − gyz )(z) = 0, for
each z ∈ X there exists δ(z) > 0 such that
gyz (x) < f (x) + for all x ∈ Bδ(z) (z).
The family of open balls {Bδ(z) (z) : z ∈ X} covers X, so it has a finite
subcover {Bδi (zi ) : 1 ≤ i ≤ n} since X is compact. By Lemma 37, the
function
gy = min{gyzi : 1 ≤ i ≤ n}
belongs to Ā. Moreover, gy (y) = f (y) and
gy (x) < f (x) + for all x ∈ X.
Next, consider gy . Since f − gy is continuous and (f − gy )(y) = 0, for
each y ∈ Y there exists δ(y) > 0 such that
gy (x) > f (x) − for all x ∈ Bδ(y) (y).
Then {Bδ(y) (y) : y ∈ X} is an open cover of X, so it has a finite subcover
{Bδ(yj ) (yj ) : 1 ≤ j ≤ m}. By Lemma 37, the function
g = max{gyj : 1 ≤ j ≤ m}
belongs to Ā. Furthermore,
f (x) − < g(x) < f (x) + for all x ∈ X,
so kf − gk∞ < , which shows that Ā is dense in C(X).
13
To complete the proof of the Stone-Weierstrass theorem, we prove several
lemmas.
Lemma 35. Let A ⊂ C(X) be a linear subspace that contains the constant
functions and separates points. If f ∈ C(X) and y, z ∈ X, then there exists
gyz ∈ A such that gyz (y) = f (y) and gyz (z) = f (z).
14
For each t ∈ [0, 1] the real sequence (qn (t)) is monotone increasing and
bounded from above by 1, so it converges to some limit q(t) as n → ∞.
Taking the limit of the recursion relations
√ as n → ∞, we find that q 2 (t) = t,
and since q(t) ≥ 0, we have q(t) = t.
According to Dini’s theorem, a monotone increasing sequence of contin-
uous functions that converges pointwise √ on a compact set to a continuous
function converges uniformly, so qn (t) → t uniformly on [0, 1].
Finally, defining the polynomials pn : [−1, 1] → R by pn (t) = qn (t2 ), we
see that pn (t) → |t| uniformly on [−1, 1].
Lemma 37. Let X be a compact metric space, and suppose that A ⊂ C(X)
is an algebra. If f, g ∈ A, then max{f, g}, min{f, g} ∈ Ā.
Proof. Since
1 1
max{f, g} = (f + g + |f − g|) , min{f, g} = (f + g − |f − g|)
2 2
it is suffices to show that |f | ∈ Ā for every f ∈ A.
If f ∈ A, then f is bounded, so f (X) ⊂ [−M, M ] for some M > 0.
From Lemma 36, there exists a sequence (pn ) of polynomials that converges
uniformly to |t| on [−1, 1]. Then pn (f /M ) ∈ A and pn (f /M ) → |f |/M
uniformly as n → ∞, since pn is uniformly continuous on [−1, 1]. It follows
that |f | ∈ Ā.
Definition 38. A metric space is separable if it has a countable dense subset.
Corollary 39. Let X ⊂ Rn be a closed, bounded set and P the set of
polynomials p : X → R. Then P is dense in (C(X), k · k∞ ). Moreover, C(X)
is separable.
Proof. A closed, bounded set in Rn is compact, and the set P of polynomials
is a subalgebra of C(X) that contains the constant functions and separates
points, so P is dense in C(X). Any polynomial can be uniformly approxi-
mated on a bounded set by a polynomial with rational coefficients, and there
are countable many such polynomials, so C(X) is separable.
In particular, we have the following special case.
Theorem 40 (Weierstrass approximation). If f : [0, 1] → R is a continuous
function and > 0, then there exists a polynomial p : [0, 1] → R such that
|f (x) − p(x)| < for every x ∈ [0, 1].
15