Exercise 4.11

Given m , we say that m is even if m2 , and m is odd otherwise.

(a)
Show that if m is odd, m = 2n + 1 for some n . [Hint: Choose n so that n < m2 < n + 1.]
(b)
Show that if p and q are odd, so are p q and pn, for any n +.
(c)
Show that if a > 0 is rational, then a = mn for some m,n + where not both n and m are even. [Hint: Let n be the smallest element of the set {xx + and x a +}.]
(d)
Theorem: 2 is irrational.

Answers

Lemma 1. If n,m and n < m, then n + 1 m and n m 1.

Proof. Suppose that n + 1 > m so that n < m < n + 1, which violates Corollary ?? since m . Thus it has to be that n + 1 m. From this it immediately follows that n = n + 1 1 m 1 by simply subtracting 1 from both sides of the previous inequality. □

Lemma 2. An integer m is even if and only if m = 2n for some integer n.

Proof. (⇒) Supposing that m is even, then n = m2 . Then clearly m = 2n.

(⇐) Now suppose that m = 2n for some integer n. Then clearly m2 = n is an integer so that m is even by definition. □

Lemma 3. An integer a is odd if and only if a2 is also odd.

Proof. (⇒) Suppose that a is odd so that a = 2n + 1 for some integer n (this is shown in part (a) below, which does not depend on this lemma). Then

a2 = a a = (2n + 1)(2n + 1) = 4n2 + 2n + 2n + 1 = 4n2 + 4n + 1 = 2 [2(n2 + n)] + 1

noting that clearly 2(n2 + n) is an integer since n is. Hence a2 is odd again by what will be shown in part (a).

(⇐) We prove this by contrapositive, so suppose that a is not odd so that it must be even. Therefore a = 2n for some integer n by Lemma 2 . Then a2 = a a = (2n)(2n) = 4n2 = 2(2n2) so that a2 is even since clearly 2n2 is an integer since n is. Thus a2 is not odd. □

Main Problem.

(a)
Here we show the converse as well, i.e. we show that m is odd if and only if m = 2n + 1 for some n .

Proof. (⇒) Suppose that m is odd so that by definition m2. It then follows from Exercise 4.9 part (b) that there is a unique integer n such that n < m2 < n + 1. We then have that 2n < m < 2(n + 1) = 2n + 2 since obviously 2 > 0. Hence by Lemma 1 we have that 2n + 1 m and also m 2n + 2 1 = 2n + 1. Therefore it has to be that m = 2n + 1 as desired.

(⇐) Now suppose that there is an n such that m = 2n + 1. Then we have that

m 2 = 2n + 1 2 = n + 1 2.

We then clearly have that n = n + 0 < n + 12 < n + 1 since 0 < 12 < 1 so that m2 = n + 12 cannot be an integer by Corollary ?? . Hence m is odd by definition. □

(b)

Proof. Suppose that p and q are odd so that p = 2k + 1 and q = 2m + 1 for some k,m by part (a). We then have that

p q = (2k + 1)(2m + 1) = 4km + 2m + 2k + 1 = 2(2km + m + k) + 1

so that p q is odd by what was shown in part (a) since clearly 2km + m + k by Exercise 4.5 since k and m are integers.

Now we show by induction on n that pn is odd for any n +. First, for n = 1 we clearly have pn = p1 = p is odd by supposition. Then, if we assume that pn is odd, we have that the product pn+1 = pn p is odd as well by what was just shown since both pn and p are odd. This completes the induction. □

(c)

Proof. Suppose that a > 0 is rational. Then a = pq for some integers p and q. Clearly it cannot be that q = 0, and if q < 0 then q = b for some b +. Then we have a = pq = p(b) = (p)b so that ab = p. Furthermore, since a and b are both positive, we have that ab = p is positive by Exercise 4.2 part (h). Thus clearly p + since p .

Now, let X = {x +ax +}. Since we just showed that b + and ab = p + it follows that b X. Since clearly X + and X is nonempty (since b X), it has a smallest element n by the well-ordering property. Letting m = an, we clearly have that m + since n X. Then, we have a = mn, noting again that m,n +.

To show that not both m and n are even, suppose to the contrary that they are both even. Then by Lemma 2 we have that m = 2k and n = 2l for some k,l . Clearly then k = m2 and l = n2 so that both k and l are positive by Exercise 4.2 part (h) since m and n (and 12) are. Hence k,l +. We have a = mn = 2k2l = kl so that al = k, which implies that l X since l and al = k are both in +. However, we also have that l = n2 < n since n > 0, which contradicts the fact that n is the smallest element of X. Thus it has to be the case that not both m and n are even. □

(d)
This is one of the most famous proofs in all of mathematics, and is often used as an example of mathematical proofs since it can be understood by most laymen.

Proof. Obviously we take 2 to be the unique positive real number such that (2)2 = 2 as was shown to exist in Exercise 4.10. Suppose to the contrary that 2 is rational so that 2 = ab for a,b + where not both a and b are even by part (c) since 2 > 0. We therefore have that 2 = (2)2 = (ab)2 = a2b2 so that 2b2 = a2. Since b2 is an integer (clearly, since b is and b2 = b b) it follows from Lemma 2 that a2 is even. This means that a itself is even by Lemma 3 . Hence a = 2n for some integer n so that a2 = (2n)2 = 4n2. From before, we then have 2b2 = a2 = 4n2 so that clearly b2 = 2n2, from which it follows as before that b2 and therefore b itself is even by Lemmas 2 and 3 . However, this is a contradiction since we previously established that a and b cannot both be even! So it has to be that 2 is not rational and is therefore irrational as desired. □

User profile picture
2019-12-01 00:00
Comments