Solution:
Every convergent sequence is bounded.
Proof. Let (xn) be a sequence which converges to ℓ , and let ϵ=1 and note that ϵ>0 . By the definition of convergence of a sequence, there exists some N∈N such that if n≥N , then ∣xn−ℓ∣<ϵ . We compute
⟹⟹∣xn−ℓ∣<ϵ⟹−ϵ<xn−ℓ<ϵ−ϵ+ℓ<xn<ϵ+ℓℓ−1<xn<ℓ+1
We make the following two calculations.
ℓ⟹ℓ+1≤∣ℓ∣≤∣ℓ∣+1
and
−ℓ⟹−∣ℓ∣⟹−∣ℓ∣−1≤∣ℓ∣≤ℓ≤ℓ−1
Therefore, we can compute
−∣ℓ∣−1≤ℓ−1<xn<ℓ+1≤∣ℓ+1⟹−∣ℓ∣−1<xn<∣ℓ+1⟹∣xn∣<∣ℓ∣+1
Let M=max{∣x1∣,∣x2∣,…,∣xN−1∣,∣ℓ∣+1} . Then given any xn , if n<N,∣xn∣≤M , and if n≥N , then
∣xn∣<∣ℓ∣+1≤M.
Hence the sequence (xn) is bounded by M.
Next: If a sequence converges then all subsequences converge and all convergent subsequences converge to the same limit.
Proof: Let {an}n∈N be any convergent sequence. Denote the limit by ℓ . Let {bn}n∈N be any subsequence. Let ε>0 be given. By the definition of convergence for {an}n∈N there exists N∈N such that ∣an−ℓ∣<ε for all n≥N . But this value N will also work for {bn}n∈N . This is because if n≥N, then bn=am for some m≥n≥N and so ∣bn−ℓ∣=∣am−ℓ∣<ε . Thus ∣bn−ℓ∣<ε for all n≥N
as required.
Comments