Mid Sem Proofs
Mid Sem Proofs
Proof. By distributivity:
a · (0 + 0) = a · 0 + a · 0
a·0=a·0+a·0
a · 0 + (−a · 0) = (a · 0 + a · 0) + (−a · 0)
0 = (a · 0 + a · 0) + (−a · 0)
0 = a · 0 + (a · 0 + (−a · 0))
0=a·0+0
0=a·0
By commutativity, a · 0 = 0 · a = 0.
1
3 Triangle inequality
Theorem 3. If a, b ∈ R, then |a + b| ≤ |a| + |b|.
|a + b|2 = (a + b)2
= a2 + 2ab + b2
≤ |a|2 + 2|a||b| + |b|2
= (|a| + |b|)2
|a − b| = |a − an + an − b|
= |(a − an ) + (an − b)|
≤ |a − an | + |b − an |
ε ε
< + =ε
2 2
This holds for every ε > 0. Therefore, |a − b| = 0 =⇒ a = b.
2
5 Squeeze theorem for sequences
Theorem 5. Suppose (an )∞ ∞ ∞
n=1 , (bn )n=1 , (cn )n=1 are sequences such that an ≤
bn ≤ cn ∀n ∈ N and lim an = lim cn = L. Then lim bn = L.
n→∞ n→∞ n→∞
ε
Fix ε > 0. ∃N1 ∈ N such that if n ≥ N1 , then |an − L| < . Also, ∃N2 ∈ N
3
ε
such that if n ≥ N2 , then |cn − L| < . Set N = max {N1 , N2 }, so both of
3
these conditions hold. If n ≥ N , then:
Define M = max {|L| + 1, |a1 |, |a2 |, . . . , |aN −1 |, |aN |}. Clearly, |an | ≤ M ∀n ∈
N.
3
7 Convergence of a bounded monotone se-
quence
Theorem 7. Suppose (an )∞ ∞
n=1 is a monotone sequence. Then (an )n=1 con-
verges if and only if it is bounded.
Consider the case where (an )∞ n=1 has infinitely many peak points n1 <
n2 < n3 < n4 < . . . . By definition, an1 > an2 > an3 > an4 > . . . . This
subsequence (ank )∞
k=1 is therefore monotone.
Consider the case where (an )∞ n=1 has finitely many peak points k1 , k2 , k3 , . . . , kl .
Set n1 = max {k1 , k2 , k3 , . . . , kl } + 1. Clearly, n1 is not a peak point. There-
fore, ∃n2 > n1 such that an2 ≥ an1 . Clearly, n2 is also not a peak point.
∃n3 > n2 such that an3 ≥ an2 . Continuing like this, we get a monotone
increasing subseqence (ank )∞ k=1 .
9 Bolzano-Weierstrass theorem
Theorem 9. Every bounded sequence has a convergent subsequence.
4
10 Limit of the product of functions
Theorem 10. Suppose lim f (x) = l and lim g(x) = m. Then lim f (x)g(x) =
x→a x→a x→a
lm.
Proof. Fix ε > 0. We need to find a δ > 0 such that if 0 < |x − a| < δ, then
|f (x)g(x) − lm| < ε. Observe that:
Since lim f (x) = l, ∃δ1 such that if 0 < |x − a| < δ1 , then |f (x) − l| < 1.
x→a
This implies |f (x)| − |l| < 1 =⇒ |f (x)| < 1 + |l|. Also, ∃δ2 such that if
ε
0 < |x − a| < δ2 , then |g(x) − m| < . In addition, ∃δ3 such that if
2(1 + |l|)
ε
0 < |x − a| < δ3 , then |f (x) − l| < . Set δ = min {δ1 , δ2 , δ3 } so all
2(|m| + 1)
of these conditions hold. If 0 < |x − a| < δ, then:
Therefore, f is continuous at x0 .
5
12 Product rule for derivatives
Theorem 12. Suppose f, g : (a, b) → R are differentiable at x ∈ (a, b). Then
f g is differentiable at x. Moreover, (f g)0 = f 0 g + g 0 f .
f (x + h)g(x + h) − f (x)g(x)
(f g)0 (x) = lim
h→0 h
f (x + h)g(x + h) − f (x + h)g(x) + f (x + h)g(x) − f (x)g(x)
= lim
h→0
h
g(x + h) − g(x) f (x + h) − f (x)
= lim f (x + h) · + g(x) ·
h→0 h h
g(x + h) − g(x) f (x + h) − f (x)
= lim f (x + h) · lim + g(x) · lim
h→0 h→0 h h→0 h
0 0
= f (x)g (x) + g(x)f (x)
13 Rolle’s theorem
Theorem 13. Suppose f : [a, b] → R is continuous on [a, b] and differentiable
on (a, b). If f (a) = f (b), then ∃c ∈ (a, b) such that f 0 (c) = 0.
Proof. If f is a constant function, that is, f (x) = f (a) ∀x ∈ (a, b), then the
theorem is obviously true. Assume f is not a constant function. Without
loss of generality, assume ∃x0 ∈ (a, b) such that f (x0 ) > f (a) (If no such
x0 exists, then ∃x1 ∈ (a, b) such that f (x1 ) < f (a). In this case, similar
arguments can be used).
By the Extreme Value Theorem, f has a global maximum on [a, b], which
we shall call c. Since f (c) ≥ f (x0 ) > f (a) = f (b), we know c 6= a and c 6= b.
Thus, c lies in (a, b) and f 0 (c) = 0.
6
14 Mean value theorem
Theorem 14. Suppose f : [a, b] → R is continuous on [a, b] and differentiable
f (b) − f (a)
on (a, b). Then ∃c ∈ (a, b) such that f 0 (c) = .
b−a
f (b) − f (a)
Proof. Consider φ(x) = f (x) − f (a) − · (x − a). Observe that:
b−a
f (b) − f (a)
φ(a) = f (a) − f (a) − · (a − a) = 0
b−a
f (b) − f (a)
φ(b) = f (b) − f (a) − · (b − a) = 0
b−a
Applying Rolle’s Theorem to φ(x), we obtain the existence of c ∈ (a, b) such
f (b) − f (a) f (b) − f (a)
that φ0 (c) = f 0 (c) − = 0 =⇒ f 0 (c) = .
b−a b−a
Proof. Take x ∈ (a, b]. Applying the Mean Value Theorem on [a, x], we
conclude that f (x) − f (a) = f 0 (c)(x − a) for some c ∈ (a, x). Therefore, as
f 0 (c) = 0,