Sequences Course
Sequences Course
1 Generality
Definition 1. • A sequence is an application u : N → R.
• For n ∈ N, u(n) is denoted by un and is called the n-th term or general term of the
sequence.
1
1.1 Bounded sequences
∃M ∈ R, ∀n ∈ N, |un | 6 M.
1
Example 2. 1. The sequence un = is bounded, ∀n ∈ N∗ (M = 1 suffices).
n
2. The sequence ((−1)n )n∈N is bounded because, |(−1)n | = 1.
• increasing if ∀n ∈ N un+1 ≥ un .
• decreasing if ∀n ∈ N un+1 ≤ un .
2
2 Convergence of a sequence
Definition 4 (Finite limit). A sequence (un )n is said to converge to a number ` if and
only if
∀ε > 0, ∃n0 ∈ N, ∀n ∈ N, (n > n0 ⇒ |un − `| < ε)
This means that for any neighborhood of l from a certain rank, the Un terms are in the
neighborhood.
If the limit ` is unique, we write lim un = `.
n−→+∞
2n + 1
∀n ∈ N, un =
n+1
Let’s show that lim un = 2. Let ε > 0, show that there exists n0 ∈ N, such that for any
n→+∞
0
integer n, n > n ⇒ |un − 2| < ε. We have
2n + 1 −1 1
|un − 2| = −2 = =
n+1 n+1 n+1
Thus
1 1 1
|un − 2| < ε ⇔ <ε⇔n+1> ⇔n> −1 (1.1)
n+1 ε ε
We set n0 = − 1 + 1 = 1ε . Therefore, for any integer n, if n > n0 = 1ε , we’ll have
1
ε
1
n> ε
− 1, so from (1), |un − 2| < ε. Hence (un )n is convergent.
3
Remark 2. A sequence that converges is said to be convergent. Otherwise, we say the
sequence diverges or that it is divergent.
Proof. We proceed by contradiction. Let (un )n∈N be a convergent sequence with two limits
|` − `0 |
` 6= `0 . Let’s choose > 0 such that < . Since lim un = `, there exists N1 such
2 n→+∞
that n > N1 implies |un − `| < . Similarly limn→+∞ un = `0 , there exists N2 such that
n > N2 implies |un − `0 | < . Let N = max (N1 , N2 ), then for this N we have:
Example 7. The following sequence ((−1)n )n∈N = (1, −1, 1, −1, ...) does not converge to
any real number.
4
3 Further Useful Results
In this section we go over some basic results about the limits of sequences.
Remark 3. The condition given in the previous result is necessary but not sufficient. For
example, the sequence ((−1)n ) is a bounded sequence but it does not converge.
Theorem 3. Suppose (un ) is a bounded and increasing sequence. Then the least upper
bound of the set {un : n ∈ N} is the limit of (un ).
Proof. Suppose sup un = M . Then for given > 0, there exists n0 such that M − ≤ un0 .
n
Since (un ) is increasing, we have un0 ≤ un for all n ≥ n0 . This implies that
M − ≤ un ≤ M ≤ M + for all n ≥ n0 .
That is un → M .
5
For decreasing sequences we have the following result and its proof is similar.
Theorem 4. Suppose (un ) is a bounded and decreasing sequence. Then the greatest lower
bound of the set {un : n ∈ N} is the limit of (un ).
1 1
2. Let (un ) and (vn ) be the following sequences un = and vn = , we have
n+1 n+2
vn < un for all n ∈ N but the two limits are equal to 0.
Theorem 6 (Squeeze Theorem or Sandwich rule). Suppose that {un }n∈N , {vn }n∈N , and
{ωn }n∈N , are sequences of real numbers such that
1. ∀n ∈ N un ≤ ωn ≤ vn
2. lim un = vn = `.
n→+∞
Then lim ωn = `
n→+∞
Proof. Let ε > 0. Since (un )n and (vn )n converge to `, there exist n1 , n2 ∈ N such that
This implies
−ε < un − ` ≤ ωn − ` ≤ vn − ` < ε
⇒ |ωn − `| < ε
So (ωn )n converges to `.
6
Example 9. (1) Let us consider the following sequence
cos n
vn = , for all n ∈ N∗ .
n
−1 cos n 1 −1 1
We have −1 ≤ cos n ≤ 1 then ≤ ≤ . Since lim = lim = 0 then
n n n n→+∞ n n→+∞ n
cos n
lim = 0.
n→+∞ n
1! + 2! + · · · + n!
Un =
(n + 2)!
For all k = 1, n,
n
X n
X n
X
k! ≤ n! ⇒ k! ≤ n! = n! 1 = nn!
k=1 k=1 k=1
so
n.n! n
0 < un ≤ =
(n + 2)! (n + 2)(n + 1)
Applying the previous theorem, we obtain
lim un = 0.
n→+∞
Proof. Let ε > 0. Since lim un = `, there exists an integer n0 such that
n→+∞
Remark 4. The converse is in general wrong. Taking the previous example, let’s consider
the sequence (un )n defined by un = (−1)n . We have lim |un | = 1, but the limit of (un )n
n→+∞
does not exist.
7
Proposition 8. Let (un )n , (vn )n be two sequences such that (un )n is bounded and lim vn =
n→+∞
0 . Then lim un vn = 0.
n→+∞
Proof. The sequence (un )n is bounded, so we can find an réel M > 0 such that ∀n ∈
N, |un | ≤ M . Let ε0 = ε
M
> 0; since vn → 0, there exists n0 ∈ N such that
ε
∀n ∈ N, n > n0 ⇒ |vn | < ε0 =
M
So
ε
∀n ∈ N, n > n0 ⇒ |un vn | ≤ |un | |vn | ≤ M = ε.
M
Hence lim un vn = 0.
n→+∞
n sin(n!)
Example 10. Let (un )n be a sequence defined by un = 2 .
n +1
n
We set vn = sin(n!) and ωn = 2 , since vn = sin(n!) is bouneded and
n +1
n 1
lim ωn = lim = lim 1 = 0.
n→+∞ n→+∞ n2 + 1 n→+∞ n +
n
Therefore lim un = 0.
n→+∞
8
` · k if `, k ∈ R,
+∞ if ` > 0 and k = +∞ or ` = +∞ and k > 0
3) lim (un · vn ) = or ` < 0 and k = −∞ or ` = −∞ and k < 0
n→+∞
−∞ if ` > 0 and k = −∞ or ` = −∞ and k > 0
or ` < 0 and k = +∞ or ` = +∞ and k < 0
`
if ` ∈ R and k ∈ R∗ ,
k
+∞ if ` > 0 and k = 0+ or ` < 0 if k = 0− or
un
4) lim = ` = +∞ and k > 0 or ` = −∞ if k < 0,
n→+∞ vn
−∞ if ` < 0 and k = 0+ or ` > 0 if k = 0−
` = −∞ and k > 0 or ` = +∞ if k < 0.
There is another useful way we can express all these rules: If (an ) and (bn ) are con-
vergent then
9
Example 11. In full detail
1 + n12 6 − n1
(n2 + 1) (6n − 1)
lim = lim
n→∞ 2n3 + 5 n→∞ 2 + n53
using the Quotient Rule
1 1
lim 1+ 2 6−
n→∞ n n
=
5
lim 2 + 3
n→∞ n
using the Product and Sum Rules
1 1
1 + lim 2
6 − lim
n→∞ n n→∞ n
=
1
2 + 5 lim
n→∞ n3
(1 + 0)(6 − 0)
=
2+0
=3
Unless you are asked to show where you use each of the rules you can keep your solutions
simpler. Either of the following is fine:
1 + n12 6 − n1
(n2 + 1) (6n − 1) (1 + 0)(6 − 0)
lim = lim 5 = =3
n→∞ 2n3 + 5 n→∞ 2 + n3 2+0
Remark 5. By induction, the Sum and Product Rules can be extended to cope with any
finite number of convergent sequences. For example, for three sequences:
5 Subsequences
Definition 6. Let (un )n∈N be a sequence. A subsequence (vn )n∈N of (un )n∈N is defined by
a function ϕ : N → N such that φ is strictly increasing and vn = uφ(n) for n ∈ N.
In other words, a subsequence is a sequence (vn )n∈N , where each vn is in (un ), and the
terms are in the right order.
10
• 2, 4, 8, 16, . . . the subsequence (u2n )
The following are not subsequences of (un ).
• 6, 4, 8, . . . the terms are not in the right order
• 2, 4, 0, . . . not all the terms are in (un )
• 1, 2, 3, . . . , 2020 finite so not a sequence.
Exercise 1. Let un = n2 . Write down the first four terms of the three subsequences
(un+4 ), (u3n−1 ) and (u2n ).
Remark 6. (1) So if (un ) is a sequence, and it has two subsequences that tend to different
limits, then (un ) does not converge. This follows from Proposition 16, and can be a useful
strategy for showing that a sequence does not converge.
(2) A sequence (un )n is convergent if and only if the subsequences (u2n ) and (u2n+1 ) are
convergent and have the same limit.
Example 13. The divergent sequence ((−1)n )n∈N admits the following convergent subse-
quences u2n = 1, u2n+1 = −1 for all n ∈ N.
6 Adjacent sequences
Definition 7. Let (un ) (vn ) be two real sequences. We say that the two sequences are
adjacent if the first is increasing, the second is decreasing, and their difference converges
to 0. In other words
1) The sequence (un ) is increasing and the sequence (vn ) is decreasing,
2) The difference (vn − un ) converges to 0, when n approaches +∞.
Theorem 11. Two adjacent sequences converge, and converge to the same limit.
Proof. We have
u0 6 u1 6 u2 6 · · · 6 un 6 · · · · · · 6 vn 6 · · · 6 v2 6 v1 6 v0
11
The sequence (un )n∈N is increasing and bounded above by v0 , so it converges to a limit `.
The sequence (vn )n∈N is decreasing and bounded below by u0 , so it converges to a limit
`0 . Therefore `0 − ` = lim (vn − un ) = 0, hence `0 = `.
n→+∞
Example 14. Let (un )n and (vn )n be two sequences defined by, ∀n ∈ N∗ ,
n
1 1 1 1 X 1
un = + + = . . . =
1! 2! 3! n! k=1 k!
1
textandvn = un +
n.n!
We have a, ∀n ∈ N∗ ,
n+1 n
X 1 X 1
un+1 − un = −
k=1
k! k=1 k!
1 1 1 1 1
= 1 + + ··· + + − 1 + + ··· +
2! n! (n + 1)! 2! n!
1
= >0
(n + 1)!
1 1
vn+1 − vn = un+1 + − un −
(n + 1) · (n + 1)! n · n!
1 1 1
= + −
(n + 1)! (n + 1) · (n + 1)! n · n!
1 1 1
= + −
(n + 1) · n! (n + 1) · (n + 1) · n! n · n!
n(n + 1) n (n + 1)2
vn+1 − vn = = + −
(n + 1)2 · n · n! (n + 1)2 · n · n! (n + 1)2 · n · n!
n(n + 1) + n − (n + 1)2
=
(n + 1)2 · n · n!
−1
= <0
(n + 1)2 · n · n!
So (vn )n is strictly decreasing. Furthermore, we have
−1
lim (un − vn ) = lim =0
n→+∞ n→+∞ n · n!
1
Moreover, it is clear that un ≤ vn (because we have vn = un + n·n!
). Hence (un )n and
(vn )n are adjacent.
12
7 Recursive Formulas for Sequences
Definition 8. Let f : I ⊂ R → R. A recursive sequence is a sequence in which terms
are defined using one or more previous terms which are given by u0 ∈ I and the relation
∀n ∈ N : un+1 = f (un )
We suppose that f (I) ⊂ I, and so the sequence is well defined.
√ √
Example 15. Let un+1 = un + 1, u0 = 1, we have f (x) = x + 1, D = [−1, +∞[ et
f (I) = [0, +∞ [⊂ I . Thus un is well defined.
Theorem 12. Let {un } be a real sequence recursively defined by un+1 = f (un ).
1. If f is increasing then the sequence (un ) is monotone. More precisely (un ) is mono-
tone:
1. Show that 0 ≤ un ≤ 3, ∀n ∈ N.
2. Study the monotonicity and the convergence of the sequence (un )n . Find its limit.
Exercise 2 (Final Exam Review 2022, Lic Math). Consider the sequence (un )n defined
2
by u0 = 1; un+1 = 1 + , n ∈ N.
1 + un
13
1. Show that 1 ≤ un ≤ 3, ∀n ∈ N.
ii) we suppose that P(n) is true and show P(n + 1). We have
1 ≤ un ≤ 3 ⇒2 ≤ 1 + un ≤ 4
1 1 1
⇒ ≤ ≤
4 1 + un 2
2 2
⇒ ≤ ≤1
4 1 + un
3 2
⇒ ≤ +1≤2
2 1 + un
2
⇒1≤ +1≤3
1 + un
Hence
1 ≤ un+1 ≤ 3.
−2
f 0 (x) = < 0,
(x + 1)2
14
4) The subsequences (u2n )n and (u2n+1 )n converge to a fixed point f ◦ f .
Calculate the fixed points of g = f ◦ f (` = lim u2n and ` = lim u2n+1 )
n→+∞ n→+∞
For all ` ∈ [1; 3] ` = g(`) = (f ◦ f )(`). We have
2 3 + 2`
g(`) = f (f (`)) = 1 + 2 =
1 + (1 + 1+`
) 2+`
So
3 + 2` √ √
g(`) = ` ⇔ = ` ⇔ 3 + 2` = `2 + 2` ⇔ ` = 3 or ` = − 3
2+`
Since the subsequences (u2n ) and (u2n+1 ) converge to the same limit ` then the sequence
(un )n also converges to ` (the two subsequences (u2n )n and (u2n+1 )n are positive, then their
√ √
limits are also positive, so the only possible limit is equal to 3). Hence lim un = 3.
n→+∞
8 Cauchy sequences
Is it possible to know whether a sequence converges (to a finite limit) without knowing
its limit? The notion of a Cauchy sequence answers this question. It reflects the intuitive
idea that the terms of a convergent sequence must be close to each other from a certain
rank
1 n
Example 17. 1) The geometric sequence 2 n∈N
is a Cauchy sequence.
We have, for p > q > 0,
p q q p−q q p−q !
1 1 1 1 1 1
− = −1 < because −1 <1
2 2 2 2 2 2
So q
1 ln
<⇒q> .
2 − ln 2
15
Taking
ln
n0 = + 1.
− ln 2
1 n
Then 2 n∈N
is a Cauchy sequence.
sin 1 sin 2 sin n
2) The sequence un = + 2 · + n is a Cauchy sequence.
2 2 2
If p > q, we have
1
Hence ∀ε > 0 choosing n0 ∈ N such that < ε. So (un )n is a Cauchy sequence.
2n0
Remark 7. To show that a sequence (Un )n is not Cauchy, we need to find some ε > 0,
so that for each n0 ∈ N there are some p, q ≥ n0 with |Up − Uq | ≥ 0.
Example 18. (a) Let (un = (−1)n ) and let ε = 1. For each n0 ∈ N, we put p = 2n0 and
q = 2n0 + 1. Note that |(−1)p − (−1)q | = |1 − (−1)| = 2 > ε. Therefore, ((−1)n ) is not
Cauchy.
(−1)n
(b) Let un = n + n
, and let ε = 1. For each n0 ∈ N, we put p = 2n0 + 2 and
q = 2n0 + 1. Then,
1 1
|up − uq | = 2n0 + 2 + − 2n0 + 1 −
2n0 + 2 2n0 + 1
1 1
=1+ +
2n0 + 2 2n0 + 1
>ε
16
(c) Let xn = ln n, and let ε = ln 2. For each n0 ∈ N, we put p = 2n0 and q = n0 . Then,
we have
|xp − xq | = | ln(2n0 ) − ln n0 | = ln 2 = ε
• The proof of the converse of the theorem is very long and technical, we refer the reader
to “Eléments d’analyse de Kada Allab” for a proof.
4. Let A = {un , n ∈ N}. Determine, whenever these exist, sup A, inf A, min A and
max A.
17