Week 02 - Real Numbers PDF
Week 02 - Real Numbers PDF
Axiomatic Foundation of R
The set R comes equipped with two binary operations denoted by + (addition) and ·
(multiplication). Let a, b,and c be real numbers. Note that R is closed under the two
binary operations, i.e. a + b ∈ R and ab ∈ R. Further, the above operations satisfy the
following properties.
M4. Existence of an multiplicative Inverse. If a 6= 0, then there exists a−1 ∈ R such that
a · a−1 = 1; a−1 is called the multiplicative inverse of a.
(c) If a ∈ R, then a · 0 = 0.
Proof. We prove (a). Using A3, A4, A2, and the hypothesis z + a = a, and A4, we have
16 RSH20150131012100
The Real Numbers R
MA313 Online 2.1 Algebraic Properties of R
Proof. We prove (a). Using M3, M4, M2, the hypothesis ab = 1, and M3, we get
The set P of positive real numbers is a subset of R with the following properties.
(i) If a, b ∈ P, then a + b ∈ P.
(ii) If a, b ∈ P, then ab ∈ P.
Properties (i) and (ii) are closure properties, i.e. the sum and product of positive real numbers
are positive. The last property simply says that for any real number, it is either positive, zero,
or ‘non–positive and is normally referred to as the Trichotomy Property.
The following are more properties of R which you should be familiar with.
Proof. We prove the first two and leave the rest as exercises.
(i)
a+c = b+c
a + c + (−c) = b + c + (−c)
a + (c + (−c)) = b + (c + (−c)) by A1
a+0 = b + 0 by A4
a = b
17 RSH20150131012100
The Real Numbers R
MA313 Online 2.2 Ordering in R
a0 + 0 = a0 + a0
Therefore, by (i), a0 = 0.
2. Solve the following equations, justifying each step by referring to an appropriate property
or theorem.
(a) 3x − 6 = 9. (c) x2 − 3 = 1.
(b) x2 = 4x. (d) (x − 3)(x + 2) = 0.
2.2 Ordering in R
Now that we have a ‘vague’ idea what the set of real numbers is, let us give it some sense of
ordering.
We write a ≤ b and read ‘a is less than or equal to b’ (or ‘b is greater than or equal
to a’) to mean that ‘b − a ∈ P ∪ {0}’.
18 RSH20150131012100
The Real Numbers R
MA313 Online 2.2 Ordering in R
Ordering Axioms in R
Let a, b, c ∈ R. The set Q, and hence R, has an order structure ≤ satisfying the following.
O1. Either a ≤ b or b ≤ a.
O4. If a ≤ b, then a + c ≤ b + c.
Proof. We prove the first three and leave the rest as exercises.
a ≤ b
a + [(−a) + (−b)] ≤ b + [(−a) + (−b)]
[a + (−a)] + (−b) ≤ [b + (−b)] + (−a)
0 + (−b) ≤ 0 + (−a)
−b ≤ −a
a ≤ b
(−c)a ≤ (−c)b
−(ac) ≤ −(bc)
bc ≤ ac by (i)
19 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Absolute Value
The distance between real numbers a and b is the absolute value |a − b| or |b − a|.
R
a b
|b − a| = |a − b|
The next result gives basic properties of the absolute value function.
(i) |a| ≥ 0
20 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Absolute Value
Proof. The proof of (i) is direct from the definition whereas the last two are routine computa-
tions.
|ab| = ab = |a||b|.
Case 2: If a ≥ 0 and b ≤ 0, then |a| = a, |b| = −b, and |ab| = −ab. Hence
Case 3: If a ≤ 0 and b ≥ 0, then |a| = −a, |b| = b, and |ab| = −ab. Hence
Case 4: If a ≤ 0 and b ≤ 0, then |a| = −a, |b| = −b, and |ab| = ab. Hence
21 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Absolute Value
Proof. Exercise.
Theorem 2.8 Let a ∈ R. If x belongs to the neighbourhood Vǫ (a) for all ǫ > 0, then x = a.
Proof. Exercise.
22 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Completeness in R
for all x1 , x2 , . . . , xn ∈ R.
6. Let ǫ > 0, δ > 0, and x ∈ R. Show that Vǫ (x) ∩ Vδ (x) and Vǫ (x) ∪ Vδ (x) are γ–
neighbourhoods of x for some appropriate values of γ.
2.4 Completeness of R
In this section we introduce and discuss the well known ‘Completeness Axiom’ which is one of
the most important principles in real analysis but first we need some definitions and preliminary
notes.
If S is nonempty and finite, then S is bounded; among the members of S there must be
a largest, denoted by max{S}, the maximum of S, and smallest, denoted by min{S}, the
minimum of S. Both the maximum and minimum of S are in S. Infinite sets may or may
not have a maximum and/or minimum.
23 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Completeness in R
Let S ⊂ R be bounded from above. A real number a is the least upper bound , or
supremum, for S if a is an upper bound for S having the property that if b is an upper
bound for S, then a ≤ b; we write
lub S = a or sup S = a.
Let S ⊂ R be bounded from below. A real number a is the greatest lower bound , or
infimum, for S if a is lower bound for S having the property that if b is a lower bound
for S, then a ≥ b; we write
glb S = a or inf S = a.
Example 2.1 Let A = [0, 2], B = (0, 2), C = [0, +∞), and D = (−∞, 0]. Then:
• min A = min C = 0;
• max A = 2, max D = 0;
• lub A = lub B = 2;
Example 2.2 It is not hard to see that b = lub(a, b) = lub[a, b] and a = inf(a, b) = inf[a, b]
for any open interval (a, b) and closed interval [a, b]. ,
Example 2.3 For the set of natural numbers N, inf N = 1 and sup N = +∞. ,
Note if M is an upper bound for S then any number greater than M is also an upper bound.
Similarly if m is a lower bound for S then any number less than m is also a lower bound.
Lemma 2.9 A number u is the supremum of a nonempty subset S of R if and only if u satisfies
the conditions:
24 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Completeness in R
Proof. Exercise.
Proof. (i)⇒(ii)
(i) If S has a smallest element, then this smallest element is the infimum of S.
(ii) If S has a greatest element, then this greatest element is the supremum of S.
Proof. (i) Let m be the smallest element of S. Then m is a lower bound of S since m ≤ s for
all s ∈ S. Suppose that m ′ is a lower bound of S. Then m ′ ≤ s for all s ∈ S. Thus m ′ ≤ m and
hence m = inf S.
We now state one of the most fundamental properties of R which is normally adopted as an
axiom. It is is also known as the Least Upper Bound Principle.
The Completeness [Supremum] Property of R: Every nonempty set of real numbers that
has an upper bound also has a supremum.
25 RSH20150131012100
The Real Numbers R
MA313 Online 2.3 Completeness in R
Proof. For if b and b ′ are two distinct suprema of S, then, assuming without loss of generality
that b ′ < b, we see, from the fact that b is a supremum of S, that there exists s ∈ S with s > b ′ ,
contradicting the fact that b ′ is a supremum of S. Thus we may properly refer to “the” supremum
of a set S if that supremum exists.
Theorem 2.13 If S ⊂ R is a nonempty and is bounded below, then it has a unique greatest lower
bound.
Proof. Write T = {−x : x ∈ S}. Let m be a lower bound for S. For each x ∈ S we have x ≥ m
and therefore −x ≤ −m; so −m is an upper bound for T . By the least–upper–bound principle,
T has a least upper bound, say b. We claim that
To prove (i), observe that for each x ∈ S we have −x ≤ b and therefore x ≥ −b. To prove (ii),
given y > −b, we have −y < b, so, by the definition of supremum, there exists z ∈ T such that
z > −y. Then −z ∈ S and −z < y; whence y is not a lower bound for S.
Taken together, (i) and (ii) show that −b is an infimum of S. The uniqueness of the infimum of
S follows from that of the supremum of T .
1. For each set below that is bounded from above, list three upper bounds for the set. Other-
wise write “NOT BOUNDED ABOVE” or “NBA”.
(a) [0, 1] (e) n1 : n ∈ N (i) ∪∞n=1 [2n, 2n + 1]
1
(b) (0, 1) (f) {0} (j) n : n ∈ N, n is prime
(k) cos nπ
(c) {2, 7} (g) [0, 1] ∪ [2, 3] 3
:n∈N
1 1
(l) sin nπ
(d) {π, e} (h) ∩∞ n=1 − n , 1 + n 3
:n∈N
3. For each se in Exercise 1, give its supremum if it has one. Otherwise write “NO sup”.
5. Let S1 = {x ∈ R : x ≥ 0}. Show in details that the set S1 has lower bounds, but no upper
bounds. Show that inf S1 = 0.
6. Let S2 = {x ∈ R : x > 0}. Does S2 have lower bounds? Doe S2 have upper bounds? Does
inf S2 exist? Does sup S2 exist? Prove your statements.
26 RSH20150131012100
The Real Numbers R
MA313 Online 2.5 Applications of the Supremum Property
8. Let S be a nonempty subset of R that is bounded below. Prove that inf S = − sup{s : s ∈ S}.
9. Show that if A and B are bounded subsets of R, then A ∪ B is a bounded set. Show that
sup(A ∪ B) = sup{sup A, sup B}.
In the following proofs, study them carefully and try to find out where does the Supremum
Property is being applied.
sup(a + S) = a + sup S.
In the proof to come, we make use of the property x = y if and only if x ≤ y and y ≤ x. This is
just a fancy way of taking about ‘equality’ of two real numbers.
Note that in the preceding proof, we make use of the ordering property of real numbers that if
x ≤ y and y ≥ x, then x = y.
27 RSH20150131012100
The Real Numbers R
MA313 Online 2.5 Applications of the Supremum Property
Theorem 2.15 Let A and B be nonempty subsets of R with the property that
Proof.
(a) If f(x) ≤ g(x) for all x ∈ D, then sup f(x) ≤ sup g(x).
Note that for all x ∈ D,
f(x) ≤ g(x) ≤ sup g(D) ⇒ sup g(D) upper bound for f(D)
⇒ sup f(D) ≤ sup g(D).
(b) Take f(x) = x2 and g(x) = x in D = {x : 0 ≤ x ≤ 1}; f(x) ≤ g(x) for all x ∈ D. Then
Here sup f(D) ≤ sup g(D), so (a) is OK but sup f(D) ≥ inf g(D).
Note that the assumption in (a) says that “f(x) ≤ g(x) for all x ∈ D”, and it does not say
anything about the relationship between sup f(D) and inf g(D).
(c) If f(x) ≤ g(y) for all x, y ∈ D, then sup f(D) ≤ inf g(D). ,
Theorem 2.16 (Archimedean Property) If x ∈ R, then there exists n ∈ N such that x < n.
28 RSH20150131012100
The Real Numbers R
MA313 Online 2.5 Applications of the Supremum Property
Proof. (Contradiction) We give a sketch of the actual proof. Suppose that n ≤ x for all n ∈ N.
Then x is an upper bound of N. By the Completeness Property, N has a supremum u ∈ R.
Hence u − 1 (being less than u) cannot be an upper bound. So there exists m ∈ N such that
u − 1 < m < u. Thus, u < m + 1 ∈ N, a contradiction.
A variation of the Archimedean Property also states that: If a and b be positive real numbers,
then there exists n ∈ N such that na > b.
Proof. Exercise.
The proof of the next result is an illustration of how the Completeness Axiom could be used to
establish that there is real number whose square is 2.
Proof. The actual proof is quite involved but we give a sketch of the main idea and how the
Completeness Axiom comes into the picture.
Consider the set S = s ∈ R : s ≥ 0, s2 < 2 . Clearly the set is nonempty since 1 ∈ S. Further,
S is bounded from above by 2 because if t > 2, then t2 > 4 so that t ∈ / S. Therefore, by the
Completeness Axiom, the supremum x = sup S exists; clearly x > 1. The rest of the proof is
basically to show that x2 = 2 by ruling out the other two possibilities x2 < 2 and x2 > 2.
We now prove that the set of rational numbers is dense in the set of real numbers. In other words,
between any two real numbers, there is always a rational number.
Theorem 2.19 (Density) Let x, y ∈ R be such that x < y. Then there exists q ∈ Q such that
x < q < y.
29 RSH20150131012100
The Real Numbers R
MA313 Online 2.5 Applications of the Supremum Property
(i) Assume 0 < x < y. Then, by Corollary (a) to the Archimedean Property, there exists n ∈ N
such that
1
0 < < y − x ⇒ 0 < nx < ny − 1. (1)
n
Furthermore, there exists m ∈ N such that
m
m − 1 ≤ nx < m ⇒ x< . (2)
n
Finally, by (1) and (2),
m
m − 1 < ny − 1 ⇒ < y. (3)
n
m
Therefore, by (2) and (3), x < < y.
n
(ii) Note that 0 < −y < −x. Then apply (i) to conclude there exists a rational number q such
that 0 < −y < q < −x which in turn x < −q < y < 0.
(iii) Considering 0 being a rational number would do, i.e. x < 0 < y.
1. Show that sup 1 − n1 : n ∈ N = 1.
2. If S = n1 − m1 : m, n ∈ N , find inf S and sup S.
(a) Let a > 0, and let aS = {as : s ∈ S}. Prove that inf(aS) = a inf S and sup(aS) =
a sup S.
(b) Let b < 0 and let bS = {bs : s ∈ S}. Prove that inf(bS) = b sup S and sup(bS) =
b inf S.
(a) For each x ∈ X, find f(x) = sup{h(x, y) : y ∈ Y}; then find inf{f(x) : x ∈ X}.
(b) For each y ∈ Y, find g(y) = inf{h(x, y) : x ∈ X}; then find sup{g(y) : y ∈ Y}. Compare
with result found in part (a).
7. Prove: If x, y ∈ Q with x < y, then there exists an irrational number z such that x < z < y.
Hint: Apply the Density Theorem.
30 RSH20150131012100
The Real Numbers R
MA313 Online 2.5 Applications of the Supremum Property
31 RSH20150131012100