Constructia multimilor de numere.pdf

  • Upload
    naparca

  • View
    237

  • Download
    0

Embed Size (px)

Citation preview

  • 7/25/2019 Constructia multimilor de numere.pdf

    1/31

    CONSTRUCTION OF NUMBER SYSTEMS

    N. MOHAN KUMAR

    1. Peanos Axioms and Natural Numbers

    We start with the axioms of Peano.

    Peanos Axioms. N is a set with the following properties.

    (1) N has a distinguished element which we call 1.(2) There exists a distinguished set map : N N.(3) is one-to-one (injective).(4) There does not exist an elementn Nsuch that(n) = 1. (So,

    in particular is not surjective).(5) (Principle of Induction) LetS N such that a) 1 Sand b)

    ifn S, then(n) S. ThenS= N.

    We call such a set N to be the set of natural numbers and elementsof this set to be natural numbers.

    Lemma 1.1. Ifn N andn = 1, then there existsm N such that

    (m) =n.Proof. Consider the subset SofN defined as,

    S={n N |n = 1 or n= (m),for some m N}.

    By definition, 1 S. Ifn S, clearly (n) S, again by definitionofS. Thus by the Principle of Induction, we see that S = N. Thisproves the lemma.

    We define the operation of addition (denoted by +) by the followingtwo recursive rules.

    (1) For all n N, n+ 1 =(n).

    (2) For any n, m N, n+(m) =(n+m).Notice that by lemma 1.1, any natural number is either 1 or of the

    form (m) for some m N and thus the defintion of addition abovedoes define it for any two natural numbers n, m.

    Similarly we define multiplication on N (denoted by , or sometimesby just writing letters adjacent to each other, as usual) by the followingtwo recursive rules.

    (1) For all n N, n 1 =n.1

  • 7/25/2019 Constructia multimilor de numere.pdf

    2/31

    2 N. MOHAN KUMAR

    (2) For any n, m N, n (m) =n m+n.

    Agian, lemma 1.1 assures that this defines multiplication of any two

    natural numbers. To get a feel for how we identify this set N as ourusual number system, let me prove some of the properties we are fa-miliar with. Remember, we may use only the axioms, definitions andwhatever we have proved before to prove the successive statements.This principle should be rigidly adhered to follow our rules of logic.

    Lemma 1.2(Associativity). Ifx, y,z N, thenx+(y+z) = (x+y)+z.

    Proof. As before let us define a subset ofN as follows.

    S={z N | x, y N, x+ (y+z) = (x+y) +z}

    To prove the lemma, we must show that S= N and again we plan touse the Principle of Induction. To apply the Principle, we must checktwo things and we will check them below.

    Step 1: 1 S.For anyx, y N, we have,

    x+ (y+ 1) =x+(y) (by definition of addition)=(x+y) (by definition of addition)= (x+y) + 1 (by definition of addition)

    Thus we get 1 S.Step 2: Ifz S, then (z) S.For anyx, y N, we have

    x+ (y+(z)) =x+(y+z) (by definition of addition)=(x+ (y+z)) (by definition of addition)=((x+y) +z) (since z S)= (x+y) +(z) (by definition of addition)

    This proves the lemma.

    Lemma 1.3 (commutativity of addition). For anyx, y N, x+y =y+x.

    Proof. As always we start with a subset SofN.

    S={y N | x N, x+y =y +x}To use induction, we need to check two things. Of course, if we showS= N, we would have proved the lemma.

    Step 1: 1 S.For this we define a new subset T ofN as follows.

    T ={x N |x+ 1 = 1 +x}

    We apply induction to this set T.

  • 7/25/2019 Constructia multimilor de numere.pdf

    3/31

    CONSTRUCTION OF NUMBER SYSTEMS 3

    Step a): Clearly 1 T, since 1 + 1 = 1 + 1.Step b): Assume x T. Then

    1 +(x) =(1 +x) (by definition of addition)=(x+ 1) (sincex T)=((x)) (by definition of addition)=(x) + 1 (by definition of addition)

    Thus we see that T= N. Going back, we see that this implies 1 S.Step 2: Ify S, then (y) S.Let x N.

    x+(y) =x+ (y+ 1) (by definition of addition)= (x+y) + 1 (by associativity, proved before)

    = (y+x) + 1 (since y S)= 1 + (y+x) (since 1 S)= (1 +y) +x (by associativity)= (y+ 1) +x (since 1 S)=(y) +x (by definition of addition)

    The correct order to prove some of the remaining properties ofNafter the above is the following. (There may be other possibilities, butat least this order will work).

    (1) (Cancellative law) For any x, y,z N, ifx+z = y+ z, thenx= y.(2) (Distributive law) Ifx, y,z N then x (y+ z) = x y+x z

    and (y+z) x= y x+z x.(3) (Associative law for multiplication) For anyx, y,z N,x(yz) =

    (xy)z.(4) For any x N, 1 x= x.(5) (commutative law for multiplication) For anyx, y N,xy = yx.

    Let me prove the distributive law now. We will only prove one of them.

    Lemma 1.4(Distributive law). For allx, y,z N,x(y +z) =xy +xz.

    Proof. Again, let

    S={z N |x(y+z) =xy +xz, x, y N}

    Step 1: 1 S.

    x(y+ 1) =x(y) (by definition of addition)=xy +x (by definition of multiplication)=xy +x 1 (by definition of multiplication)

  • 7/25/2019 Constructia multimilor de numere.pdf

    4/31

    4 N. MOHAN KUMAR

    Step 2: Ifz S, then (z) S.

    x(y+(z)) =x(y+z) (by definition of addition)=x(y+z) +x (by definition of multiplication)= (xy+xz) +x (since z S)=xy + (xz+x) (by associativity of addition)=xy +x(z) (by definition of multiplication)

    Thus by Induction, S= N and we have proved the lemma.

    Exercise 1. Prove the remaining properties stated above. Remember,you may use anything proved earlier for a proof, but no later propertymay be used in the proof.

    1.1. Ordering on N. Next we introduce the ordering on N.

    Definition1. Ifn, m N, we say that n is less thanm, writtenn < m,if there exists ak N such thatm = n + k. We also writen m, readn is less than or equal to m, to mean that either n= m or n < m.

    Lemma 1.5. Ifx, y,z N andx < y andy < z thenx < z.

    Proof. The assumption x < y means y = x +k for some k N.Similarly we get z=y +l for some l N. Thus, we get,

    z= y +l

    = (x+k) +l

    =x+ (k+l) (by associativity)

    Thus by definition x < zsince k+l N.

    The same argument can be used to show the following.

    Lemma 1.6. Letx, y,z N.

    (1) Ifx y andy < z, thenx < z.(2) Ifx < y andy z, thenx < z.(3) Ifx y andy z, thenx z.

    Exercise 2. If x,y,z N and x < y show that x+ z < y +z and

    xz < yz.

    Lemma 1.7. For anym N, m=m+ 1.

    Proof. As usual define a subset S N as follows:

    S={n N |n =n+ 1}

    Clearly, 1 S, since if not, 1 = 1+1 = (1), by definition of additionand 1=(k) for any k N by Peanos axioms (number 4).

  • 7/25/2019 Constructia multimilor de numere.pdf

    5/31

    CONSTRUCTION OF NUMBER SYSTEMS 5

    Assume n S. If (n) is not in S, then (n) = (n) + 1. Thenby definition of addition, (n) = ((n)). By the third axiom, this

    means, n= (n) which in turn is n + 1 by definition of addition. Thisis impossible since n S.

    Lemma 1.8. For anym, k N, m=m+k.

    Proof. Again define a subset S N as follows:

    S={k N | m N, m=m+k}

    From the previous lemma, we see that 1 S. Ifk S, we want toshow that (k) S and then by induction we would be done. Thatis, we want to show that m = m+ (k) for any m. Notice thatm+(k) =(m+k), by definition of addition.

    Let us define a subset T as follows:

    T ={m N |m =(m+k)}

    Clearly 1 T by axiom 4. Assume m T. Want to show that(m) T. If (m) = ((m) +k), by axiom 3, we see that m =(m) +k. Thus we have,

    m= (m) +k

    = (m+ 1) +k (by definition of addition)

    =m+ (1 +k) (by associativity)

    =m+ (k+ 1) (by commutativity)=m+(k) (by definition of addition)

    =(m+k) (by definition of addition)

    But this contradicts our assumption that m T.

    Lemma 1.9 (Well ordering ofN). Ifn, m N, then exactly one of thefollowing is true. Eithern < m orn= m orm < n.

    Proof. Let us first prove only one of these can hold. Ifn < m, then bydefinition, m = n + k for some elementk N. By the previous lemma,we see that m = n. Ifm < n, then there exists an l N such thatn = m+l which implies m= (m+l) + k =m+ (l+k) which againis not possible by the previous lemma. The other cases are similar andleft as an exercise.

    To finish the proof we consider the set S, fixing an n.

    S={m N |n < m, n= m or m < n}

    Step 1: 1 S.

  • 7/25/2019 Constructia multimilor de numere.pdf

    6/31

    6 N. MOHAN KUMAR

    Ifn = 1, clearly 1 S. Ifn = 1, then by lemma 1.1, n = (k) =k+ 1 = 1 +k and thus by definition of our ordering, 1 < n.

    Step 2: IfmS then (m) S.Assume m S. This means we have three possibilities, namely

    n < m or n = m or m < n. First, let us look at the case n < m.Then m = n+k for some k. Thus(m) = (n+k) = n+(k) andso n < (m) and hence (m) S. Next possibility is n = m. Then(m) =m +1 =n +1 and thusn < (m) and again(m) S. Finally,we have the possibility ofm < n. Thusn = m+k for some elementk N. Ifk = 1, then n= (m) and thus (m) S. If not, by lemma1.1, k= (l) and thus n = m+(l) and thus,

    n= m+(l)

    m+ (l+ 1) (by definition of addition)=m+ (1 +l) (by commutativity)

    = (m+ 1) +l (by associativity)

    =(m) +l (by definition of addition).

    Therefore (m)< n by definition of our ordering and thus (m) S.Thus in any case (m) S. Therefore by induction, S= N and we aredone.

    Remark 1. As usual, we will write m > n, read mis greater than nto

    mean n < m. Similarl meaning is assigned to m n.

    Next I want to prove some alternate forms of induction which arefrequently used. We start with a definition.

    Definition 2. Let S N. Then an element n S is called a leastelement if for any m S, n m.

    Lemma 1.10. LetS N. IfShas a least element, then it is unique.So it makes sense to use the definite article the instead of a if a leastelement exists and call it the least element.

    Proof. Assume S has two least elements, say n and m. Thus we see

    that n m andm n. From the well ordering lemma, it is clear thatn= m.

    Theorem 1.1(First alternate form of Induction). IfS NandS=thenShas a least element.

    Proof. As usual let

    T ={n N |ifn S N,then Shas a least element}

  • 7/25/2019 Constructia multimilor de numere.pdf

    7/31

    CONSTRUCTION OF NUMBER SYSTEMS 7

    Caution: HereTis a fixed set defined as above. But, Sis a variablesubset ofN.

    I will leave it as an exercise to check that 1 T. Next assumethat n Tand we want to show that (n) T. So let S N with(n) S. Ifn S, then by hypothesis, we know that Shas a leastelement. So assume that n is not inSand considerA = S {n}. Thenn A and thus A has a least element by hypothesis. Let us call thisleast element a.

    There are two possibilities. Eithera = n or a = n. Ifa = n, thena S. Ifm S, then clearly m A and thus a m. So we see thata S is a least element.

    Next assume a = n. Then I claim that (n) is the least elemnt ofS. Ifm S, we know that a = n m. But n Sand thus n = m.Thus by definition of less than or equal to, we see that n < m. Thuswe may write m =n+k for some k N by defintion. Ifk = 1, thenm= n + 1 =(n). Ifk = 1, then by the first lemma, k = (l) for somel N. Thus

    m= n+ (l+ 1) =n+ (1 +l) = (n+ 1) +l = (n) +l

    and thus(n)< m. Thus we see that (n) is a least element ofSandwe are done.

    Some of you may be more familiar with the following form of induc-

    tion, though all the three are equivalent.Theorem 1.2(Second alternate form of Induction). LetP(n)be math-ematical statements forn N. Assume

    (1) P(1) is true.(2) IfP(n) is true, thenP(n+ 1) is true.

    ThenP(n) is true for alln N.

    Proof. Define a set S= {n N|P(n) is false}. We wish to show thatS=. If non-empty, by the previous form of induction,Theorem 1.1,we have a least element m S. By the first hypothesis of the theorem,m

    = 1. Thenm = p+ 1 for some p

    N. Since p < m and m being

    the least elelement ofS, we know that pSand thus P(p) is true bydefinition of the setS. Now, by our second hypothesis, P(p+1) =P(m)is true and hence m S, a contradiction, proving the result.

    Theorem 1.3 (Third alternate form of Induction). LetP(n) be math-ematical statements fosn N. Asuume,

    (1) P(1) is true.(2) Ifn >1 andP(k) is true for allk < n, thenP(n) is true.

  • 7/25/2019 Constructia multimilor de numere.pdf

    8/31

    8 N. MOHAN KUMAR

    ThenP(n) is true for alln.

    Proof. As before, let S = {n N|P(n) is false} and we wish to showthat S = . So assume that it is non-empty and let m S be theleast element assured by Theroem 1.1. Again, as before, by the firsthypothesis, 1Sand thusm >1. By minimality ofm, ifk < m, thenkSand henceP(k) is true. Thus by second hypothesisP(m) is trueand thus mS, which is a contradiction, proving the theorem.

    We will use these forms in the next section on Number Theory toprove results familiar to you. We state some more properties of naturalnumbers, which can be proved using the above ordering properties ofN.

    (1) (cancellative law for multiplication) For anyx, y,zN

    , ifxz=yzthen x = y.(2) (uniqueness of identity) For some x, y N, if xy = x, then

    y = 1.At this point, we will use our usual nomenclature for natural

    number. We already have called a special number 1 and thenwe call 2 = 1 + 1, 3 = 2 + 1 etc. in the usual fashion.

    2. Integers

    We will briefly desribe the construction of integers and rational num-bers below and state various properties in the correct order and prove

    just a few to give a flavour.Consider the set S = N N and put a relation on it as follows:

    (a, b) (c, d) if and only if a+ d = b+ c. (As usual, we denote atypical element in Sby an ordered pair of natural numbers)

    Check that this is an equivalence relation on S. Let Z be the set ofequivalence classes under this relation. Define an operation (addition)on Z as follows: If A, B Z, then recall that A, B are non-emptysubsets of S and thus we may pick elements (a, b) A and (c, d) B. With our notation for equivalence classes, this means A = [(a, b)]for example. Define an operation tentatively denoted by, to avoidconfusion, as follows:

    A B = [(a+c, b+d)]

    There is a prioria problem with this definition. To make sure thatthe operation is well-defined (a term we will see several times in thesequel), we must make sure that the right hand side above has onlyvalue. This operation is supposed to be a function fromZ Z Z,given two integers, we must get a well-defined integer as its sum. But,let us look at our definition. Here we picked some (a, b) A and

  • 7/25/2019 Constructia multimilor de numere.pdf

    9/31

    CONSTRUCTION OF NUMBER SYSTEMS 9

    (c, d) B and declared that A B = [(a+c, b+d)]. We could haveeasily picked another (a, b) A and (c, d)B . Then we would have

    gotA B to be [(a + c, b + d)], which may very well be different from[(a + c, b + d)] and then we really do not have function from ZZ Zand no real definition. So, in such situations, the first order of businessis always making sure that it is well-defined. In other words, with theabove notation, we must check that [(a+c, b+d)] = [(a +c, b +d)].For once let us check this.

    Lemma 2.1. The addition defined above is well-defined.

    Proof. As discussed, we must check that ifA = [(a, b)] = [(ab)] andB = [(c, d)] = [(c, d)], then we must check that [(a + c, b + d)] = [(a +c, b + d)]. Unwinding the defintions, this means that if (a, b)(a, b)

    and (c, d)(c, d), then we must check (a + c, b + d) (a + c, b + d).Again looking at our relation, we get that a+b =a +b and c+d =c + d. Adding them we get a + b + c + d =a + b + c + d, which impliesthat (a+c, b+d) (a +c, b +d).

    (Intuitively, the element [(a, b)] should be thought of as a b inour familiar settings though we are yet define subtraction.) Definemultiplication tentatively denoted by as follows:

    A B = [(ac+bd, ad+bc)]

    and as before make sure that this is well-defined. Now proofs of all

    the familiar properties of addition and multiplication of integers canbe carried out, by using the definitions and corresponding propertiesof natural numbers.

    (1) Associativity of addition.(2) Commutativity of addition.(3) Cancellative property of addition.(4) For any two natural number a, b N, (a, a) (b, b) and thus

    [(a, a)] = [(b, b)] whic we denote by the symbol 0. Then for anyA Z, A 0 =A = 0 A.

    (5) Additive inverse: If A = [(a, b)], then we denote by A =[(b, a)], the additive inverseofA. Then A (A) = 0.

    (6) IfAB = 0 thenB =Aand in particular the additive inverseis unique.

    (7) Distributivity.(8) Associative law for multiplication.(9) Commutative law for multiplication.

    (10) For any a, b N, ((a), a) ((b), b) and thus we denote theequivalence class [((a), a)] for any a N, by the symbol 1.Then for any A Z, A 1 =A = 1 A.

  • 7/25/2019 Constructia multimilor de numere.pdf

    10/31

    10 N. MOHAN KUMAR

    (11) Cancellative law for multiplication: IfA, B,C Z andA C=B C withC= 0, then A= B .

    (12) Uniqueness of identitiy: IfA B =A and A= 0, then B = 1.(13) A 0 = 0 for all A Z.(14) IfA B = 0, then either A= 0 or B = 0.(15) For anya, b, k N, (a + k, a) (b + k, b) and thus [(a + k, a)] =

    [(b+k, b)]. So define a mapf : N Z byf(k) = [(a+k, a)]for some a N. Then f is one-one and f(a+b) =f(a) f(b)and f(ab) =f(a) f(b).

    The last property ensures that N Z via f and the addition andmultiplication are respected by f. Thus we may now drop , andwrite just +, .

    As before we define an ordering on Z by saying that A < B ifA=[(a, b)] andB = [(c, d)], then a + d < b + c. Make sure that this is welldefined and we define A B if either A = B or A < B. Also showthat if a, b N, then a < b if and only iff(a) < f(b) and thus theordering is also respected by f. We say thatA Zis positiveif 0< Aand non-negative if 0 A. IfA < 0, we say that A is negative. Asusual, we write A > B to mean B < Aetc.

    Lemma 2.2. LetA= [(a, b)]. ThenA is positive if and only ifb < a.

    Proof. If 0 < A, then since 0 = [(a, a)], we see that a+b < a+a bydefinition of the ordering. Using the definition of ordering in N and

    cancellation, the result follows. Converse is equally easy.

    Lemma 2.3. A is positive if and only if A = f(k) for some naturalnumberk.

    Proof. Let A = [(a, b)]. First assume that it is positive. Then b < afrom the previous lemma and thus a= b+k for some natural numberk and thus A= [(b+k, b)] =f(k). Converse is equally easy.

    Lemma 2.4. A Z is positive if and only ifA is negative.

    Proof. Left as an exercise.

    Lemma 2.5. Ifa, b, c N witha < b thenac < bc.Proof. If a < b, then b = a+ k for some natural number k. Thusbc= ac+kc. Since kc N, by definition, ac < bc.

    Corollary 2.1. Ifa < b fora, b N, thena2 =a a < b2 =b b.

    Proof. From the previous lemma, since a < b, we geta2 < ab. Applyingthe lemma again, we get a b < b2. Putting them together, we geta2 < b2.

  • 7/25/2019 Constructia multimilor de numere.pdf

    11/31

    CONSTRUCTION OF NUMBER SYSTEMS 11

    Lemma 2.6. Let a, b N and 1 < a. Then there exists a naturalnumber N such that for all n N, b < an. (Recall, an is just a

    convenient way of writing the product ofa, n times).

    Proof. Consider the set

    S={b N |there exisits Nsuch thatnwithnN, b < an}

    Then 1 S. For this take N = 1 and apply the previous lemma asfollows. Let

    T ={n N|1< an}.

    Then 1 T since 1< a. Ifn T, then we have, 1< an. Multiplyingby a, from the previous lemma, we have a < an+1. Putting thesetogether, we have 1< an+1 and thus n+ 1 Tand thus by induction

    we see that T = N, proving 1 S.Assume that b S. So, there exists N such that b < an for alln N. I claim that for (b), we can take instead ofN, N+ 1. Letn N + 1. Since n = 1, we may write n = m+ 1 and m N.Thus by induction hypothesis, b < am and thus by the lemma above,ab < an. Since 1 < a, we can write a = k+ 1. Thusab = bk+ b So,ab= bk +b b+ 1. Thus we get b+ 1 < an. So b+ 1 Sand we aredone by induction.

    Let us denote by N = N {0} Z, where N is identified with the

    subsetf(N

    ). We have a mapZ

    N

    called theabsolute value, denotedby| |. |a|= a ifais non-negative and |a|= aifais negative.

    Lemma 2.7. For anya Z, we have|a| a |a|. Converseley, ifc0 is an integer andc a c, then|a| c

    Proof. First assume that a 0. Then |a| = a by defintion. So, theinequlaity we need is a a a. Sincea a by definition, we onlyneed to verify that a a. But this is same as 2a 0, by adding ato both sides of the inequality and this is clear. The case ofa < 0 isequally easy.

    To prove the second statement, we work exactly as before by looking

    at the two cases ofa 0 and a < 0. Ifa 0, then a=|a| and sincea c, we get that |a| c. Ifa

  • 7/25/2019 Constructia multimilor de numere.pdf

    12/31

    12 N. MOHAN KUMAR

    Since |a| + |b| 0, by the previous lemma. we are done.

    Finally now we can define a new operation subtractiondenoted by in Z as follows. Ifa, b Z, then a b = a+ (b). I will leave thestandard properties of subtraction to be verified by the reader. Let meclose this section by yet another form of induction.

    Theorem 2.1 (Fourth alternate form of Induction). Let S Z bea non-empty subset of the integers with the property that there is anm Z such that for alla S, a > m. (That is to say that the setSis bounded below). ThenShas a least element.

    Proof. Consider the set T = {a m|a S}. Since S = nor is T.Since a > m, am > 0 and hence T N. Thus, by Theorem 1.1,

    T has a minimal element, say p. Thenq= p+m Sand we claimthat qis the least element ofS. IfaS, then a m T and hencea m p and thusa p + m= q. Thus by definition of least element,q is the least element ofS.

    Exercise 3. Show that ifa, b Z, then a (b) =(ab).

    3. Some Number Theory

    We will not use most of what we prove in this section in the sequel.I have included it only to connect our discussions with facts familiarto you and thus giving you some bearing in this abstract jungle. We

    start with one of the earliest results you might have studied in school.Theorem 3.1 (Division Algorithm). Let a, d Z withd = 0. Thenthere exists unique integersq, r Z such thata= qd+r and0 r 0. Consider the set S= {a qd|a qd 0, q Z}. First Iclaim thata + |a|d 0, showing thatS=. Ifa = 0, thena + |a|d= 0,ifa > 0, then a+ |a|d = a+ ad = a(1 +d) > 0 and if a < 0, thena+ |a|d = a ad = a(1 d) 0, since a < 0 and 1 d 0. SinceS is bounded below by zero, we can apply Theorem 2.1 to conclude

    that S has a minimal element, say 0 r = aqd for some q Z.So, a = qd+r and if we show that r < d, we would have proved theexistence part of the theorem. Ifr d, then a (q+ 1)d= r d 0.Thus r d Sand since r d < r, this contradicts the minimality ofr. So, r < d.

    Next, we prove uniqueness. If a = qd +r = qd + r with 0 r, r < d, we get (qq)d = r r. If q = q, then this impliesr =r, proving uniqueness. Ifq= q, then taking absolute values, we

  • 7/25/2019 Constructia multimilor de numere.pdf

    13/31

    CONSTRUCTION OF NUMBER SYSTEMS 13

    get, d |(q q)d| = |r r |. But since 0 r, r < d, we see that|r r|< d, which leads to a contradiction. Thus uniqueness is proved.

    Finally, ifd < 0, let e = d = |d| > 0. Thus by the previous part,we havea = qe+rwithq, r Z and 0 r < e= |d|. So,a = (q)d+ras desired.

    As usual if 0=d Z, and a Z, we say that d dividesa ifa= mdfor some m Z. Symbolically, this is written as d| a.

    Definition3. Leta, b Z with at least one of them non-zero. Then thegreatest common divisor ofa, b, written gcd(a, b) is a number d Nsatisfying the following two properties.

    (1) d| a and d| b.

    (2) Ife N divides both aand b, then e| d.Notice that gcd is defined only for two numbers with at least one

    of them non-zero. Also, notice that it is a natural number. What isnot clear from the definition is whether such a number exists and if itexists whether it is unique and these we proceed to prove.

    Lemma 3.1. Let a, b Z with at least one of them non-zero. Ifgcd(a, b) exists, then it is unique.

    Proof. Letd = gcd(a, b) ande= gcd(a, b). We wish to show thatd = e.By first property in the definition applied to e we get that e| a, e| b.

    Now applying the second property, we see that e | d. Reversing theroles, we see that d | e. It is easy to see then d = e, though let me givean explicit proof.

    e | d means we can write d = pe with p Z. Since d, e N, thisforces p > 0 and hence p N. Similalry we get e = qd with q N.Substituting, we get,d = pqd. Cancellingd >0 (which we have shownearlier), we get 1 = pq. If we show that this implies p = q= 1, wewould be done. Ifp= 1, we could write p= s + 1, s N from earlierproperties of natural numbers. Thus we getqs+q= 1. Ifq= 1, wehave d =e, so we may also assume that q >1 and thus we can writeq= t +1. Thenqs + t + 1 =(qs + t) = 1, but Peanos axioms say that

    1 is not in the image of , a contradiction, proving what we need.

    Theorem 3.2 (Existence of gcd). Let a, b Z with at least one ofthem non-zero. Thengcd(a, b) exists.

    Proof. Consider the set, S = {ma+nb > 0|m, n Z}. As usual, weclaim that this set is non-empty. Since at least one ofa, b is non-zero,we may assume that a = 0, possibly after renaming them. Then letm = a, n = 0. So,a a+ 0 b = a2 > 0 and hence a2 S. So S is

  • 7/25/2019 Constructia multimilor de numere.pdf

    14/31

    14 N. MOHAN KUMAR

    non-empty. SinceS N, by Theorem 1.1, Shas a minimal element,sayd. By definition of the set S, we havem, n Z so thatd = ma +nb.

    I claim that d = gcd(a, b).For this, we need to check the two conditions in the definition of

    gcd. The second one is easy. Ife divides both a, b, then we can writea= pe, b= qefor somep, q Z and substituting, we get,d = ma+nb=mpe+nqe = (mp+nq)e and since mp+nq Z, we see that e| d.

    For the first condition, we proceed as follows. First, we show thatd |a, the other case being similar, we shall omit it. By division algorithm,we can write a= qd+r with q, r Z and 0 r < d. Ifr = 0, d | a,so let us assume that r >0 and then we will arrive at a contradiction.Then r = a qd = a q(ma+ nb) = (1 qm)a+ (qn)b and bydefinition of the set S, we see that r S. But, r < d, contradictingthe minimality ofd.

    The above proof gives something stronger and it is in this form it isoften used, so let us state this explicitly.

    Corollary 3.1. Leta, b Z with at least one of them non-zero. Thengcd(a, b)exists and is unique. Further, it is the smallest natural numberof the formma+nb withm, n Z.

    Here is an immediate application.

    Corollary 3.2. Letp,a,b Z and assume thatp = 0. Ifp | ab and

    gcd(p, a) = 1, thenp| b.Proof. gcd(p, a) = 1 implies there exists integers m, n such that 1 =mp + na. Multiplying by b we get, b = mpb + nab. Sincep | ab, we canwriteab = spfor somes Z. Thus we get,b = mpb +nsp= (mb+ns)pand since mb+ns Z, we get that p| b.

    Definition 4. A natural number p is a prime number ifp= 1 and theonly natural numbers dividing it are 1 or p. An integer n is called acomposite number if|n| = 0, 1 and |n| is not a prime.

    I will not give examples of primes, since I am sure most of you arefamiliar with them.

    Exercise 4. (1) Show that if p is a prime then for any a N,gcd(p, a) = 1 or gcd(p, a) =p.

    (2) Show that ifp is a prime and p| ab for a, b Z, then p| a orp| b.

    (3) Show that if a prime pdivides a prime q, then p= q.(4) Show that if a primep dividesqn for a primeqandn N, then

    p= q.

  • 7/25/2019 Constructia multimilor de numere.pdf

    15/31

    CONSTRUCTION OF NUMBER SYSTEMS 15

    Theorem 3.3 (Fundamental Theorem of Arithmetic, Part 1). Let1 = n N. Then there exists primes, p1, p2, . . . , pk such that n =

    p1p2 pk. That is, anyn N, n >1 is a product of primes.

    Proof. As usual we start with the set

    S={n N|n >1, n is not a product of primes}.

    We wish to show that S is empty and if it is non-empty, we let n Sbe the least element, assured by Theorem 1.1. Now, n can not be aprime, since then n is the product of one prime. Thus by definition ofa prime, there exists a natural number d which divides n and d = 1, n.Then by properties of natural numbers, we get 1 < d < n. Sincen= defor some natural number e, we get that 1 < e < n. By minimality of

    n, we getd, eSand since they are not 1, they are product of primes.So, d= p1 pr, e= q1 qs for primes pi, qj. Thus,

    n= de = p1 pr q1 qs

    and hence n is a product of primes. So, nS, leading to the desiredcontradiction.

    Thus, ifn N and n >1, we can write n= p1 pk for primes pis.Collecting the primes and ordering them, we may assume that thereexists primes p1 1 be a natural number and let n = pa11 p

    amm as in the previous

    paragraph. Then this expression is unique. That is, if n = qb11 qbll

    withq1 1. Then p1 pj (j may be 1) and since

    pj = q1 < qi = p1, we get p1 < p1, a contradiction. So, we see thati= 1 and p1 =q1. Next we claim that a1 =b1. If not we may assume

  • 7/25/2019 Constructia multimilor de numere.pdf

    16/31

    16 N. MOHAN KUMAR

    by well ordering, that a1 > b1 (or the other way around, but we caninterchangep, q. Cancelling pb11 , we get,

    pa1b11 pa22 p

    akk =q

    b22 q

    bll .

    But then p1 = qi for some i > 1 as before, but all these are greaterthan q1 =p1, which is impossible. This proves that a1 =b1. Then wehave,

    m= pa22 pakk =q

    b22 q

    bll .

    Since m < n,mSand thus, by minimality ofn, the theorem is truefor m. This implies, k= l, pi=qi for i >1 andai = bi for i >1. Thissays, sincep1=q1and a1=b1, that the theorem is true for nand hencenS, which is the desired contradiction, proving the theorem.

    Theorem 3.5(Infinitude of primes). There are infinitely many primes.Proof. We know that there at least some primes, for example 2, 3. As-sume there are only finitley many primes, say p1, . . . , pk. Consider thenatural number N=p1p2 pk+ 1. Then clearlyN >1 and hence bythe fundamental theorem, there exists a prime number qwhich dividesN. But, since the pis are all the primes, q = pi for some i. ThuspidividesN. ThenpidividesNp1 pi pk = 1 and no prime numbercan divide 1, leading to a contradiction. This proves the theorem.

    4. Rational numbers

    The idea is the same. So, I will briefly sketch the construction. Nowconsider the set S = Z (Z {0}) and put a relation as follows.(a, b) (c, d) if ad = bc. One easily checks that this is indeed anequivalence relation on Sand the set of equivalence classes is calledthe rational numbers and denoted by Q. As usual, addition is definedby [(a, b)] [(c, d)] = [(ad+ bc, bd)] and multiplication by [(a, b)][(c, d)] = [(ac, bd)], where now we have addition and multiplicationof integers inside the brackets. As usuaul, we check that this is welldefined and all the standard properties. We also have a one-one mapf : Z Q given by f(a) = [(a, 1)] and then f(a+b) = f(a) f(b)and f(ab) =f(a) f(b). Intuitively, we are thinking of [(a, b)] asa/b.

    Using f, we can identify Z as a subset ofQ in the usual way. Thusagain, we can drop , and write the usual symbols for addition andmultiplication.

    In Q, we have a new operation, division, as usual denoted by a/bfor a, b Q and b = 0. This is defined as follows: IfA = [(a, b)] andB = [(c, d)], with a,b,c,d Z, b = 0 = d, then B = 0 implies thatc= 0. Define A/B = [(ad, bc)] and make sure that this is well defined.Also notice that since both b and c are not zero, bc= 0.

  • 7/25/2019 Constructia multimilor de numere.pdf

    17/31

    CONSTRUCTION OF NUMBER SYSTEMS 17

    Lemma 4.1. IfA is any rational number, thenA= [(a, b)], for somea, b Z withb positive.

    Proof. By defintion, A = [(a, b)] with b = 0, a, b Z. Ifb is positive,then we are done. If not, we know that b is positive. One easily seesthat A= [(a, b)] and thus we are done.

    We introduce an order on Q as follows. IfA, B Q, writeA= [(a, b)]and B = [(c, d)] with b, d both positive. Then we define, A < B ifad < bc. One checks that this is well defined and has all the usualproperties. As always, writeA B to mean either A= B or A < B.Absolute value of a rational number can be defined as before, afterdefining what is positive, negative etc. Again, I will assume that we

    can prove all the usual properties of ordering onQ

    .Exercise 5. (1) Show that ifa < b are two rational numbers, then

    there exists c Q with a < c < b.(2) Prove triangle inequality (see lemma 2.8) for Q.

    5. Real Numbers

    Let me start with some observations. We started with natural num-bers which had this very important property of Induction. In otherwords, any non-empty subset had a least element. But the systemlacked operations like subtraction and thus we were forced to enlarge

    the system to integers, which had subtraction, and at least a suitableform of induction; namely, any non-empty subset which is bounded be-lowhad a minimal element. But integers still lacked division and thuswe enlarged our system to the rational numbers to rectify this lacuna.But, now, alas we have lost any semblance of the minimal elementproperty which was so important and desirable. In other words, thereare now subsets ofQ which are bounded below with no minimal ele-ment in sight. (Not just in the set, but not even in Q). So, the plan ofconstructing real numbers is to rectify this important problem with Q.

    Let me elaborate the above statement. Let

    S={x Q |x2

    >2 and xis positive}.Clearly this set is non-empty and bounded below. For example, 2 Sand ifx S, then x > 1. But I claim that this set has no minimalelement even in Q. Assume a Q is such a minimal element. Then ahas two properties. First,a x for all x S. Second, ifb Q, withb x for allx S, thenb a. I claim no such rational number exists.Since 1 works as a b, we see immediately that a 1. In particular amust be positive. I claim thata2 2. If not, a2 > 2 and a S. So

  • 7/25/2019 Constructia multimilor de numere.pdf

    18/31

    18 N. MOHAN KUMAR

    a2 = 2 + r for some positive rational number. We can choose a largenatural number N so that 2a/N < r. Consider c = a(1/N) < a.

    Thenc2 =a2 2

    a

    N +

    1

    N2 = 2 + (r 2

    a

    N) +

    1

    N2 >2.

    Thus c Sand c < a. This is a contradiction. Thus a2 2.Next I leave it as a (non-trivial) exercise that there is no rational

    number with a2 = 2 and thus we must have a2 < 2. Then againwrite 2 = a2 +r with r a positive rational number. As before we canchoose a large natural number N such that rN2a 1 and thus2a/N+ 1/N2 < r. Now considerb = a + (1/N)> a. One easily checksthat b2

  • 7/25/2019 Constructia multimilor de numere.pdf

    19/31

    CONSTRUCTION OF NUMBER SYSTEMS 19

    Exercise 6. (1) Ifa is any rational number, show that the sequencedefined as xn=a for all n N is a CS.

    (2) Let g : N N be an increasing function. That is, ifn > mthen g(n) > g(m). If {xn} is a Cauchy sequence, show that{yn} is a CS, where yn = xg(n). ({yn} is called a sub-sequenceof{xn}).

    (3) If{xn}is a CS of rational numbers, show that for any rationalnumbera, {axn}is a CS.

    Example 1. (1) Letxn = n for all n N. Then this is not a CS.As I said in the previous paragraph, we need to find just one

    positive rational number which violates the CS condition. Forthis take = 1. If anNexisted, then we must have |xn xm| 0 be given. (Hereagain, to figure out the N, one may have to work backwardsand can be tricky.) Let us do the analysis for once.

    We need an Nso that for any n, m N, we must have,

    |xn xm|= |2n 2m|< .

    Without loss of generality, we may assume that n m N.Then |2n 2m| = 2m|2mn 1|. Since 0 < 2mn 1,because n m, we see that |2mn 1| < 1 and thus we seethat |2n 2m| < 2m. But, since m N, we also have2m 2N. So, if we had 2N < , then we would be done.Notice that we finally ended up with a condition on Nand noton which n, m N we need to look at. This is usually theessence of most such arguments.

    So, we see that we only need to find an Nsuch that 2N < ,

    for the given positive . Since = 0, we have =1 Q andsince is positive so is . So, we want an Nso that 2N > . Ifwe write= a/b witha, bpositive integers, then it is clear thata . So, if we found an Nso that 2N > a, we would be done.But this is essentially the content of lemma 2.6.

    So if you want to write a proof, we invert the steps, so thatit is easy to follow the arguments. Let me do this now forillustration.

  • 7/25/2019 Constructia multimilor de numere.pdf

    20/31

    20 N. MOHAN KUMAR

    Proof. We wish to show that the sequence {xn} = {2n} is a

    CS.

    So, let >0 be a positive rational number. Then=1 Qis a positive rational number. Writing = a/b for positiveintegers a, b, we see immediatley that a . By lemma 2.6,since 2> 1, there exists anNsuch that

    2N a (1)

    Then we claim that for anyn, m N, (for theNfrom the equa-tion above) |xn xm| < , which will prove that our sequenceis a CS.

    We may assume that n m N. Then

    |xn xm|= |2

    n

    2

    m

    |= 2

    m

    |2

    mn

    1|.Since n m, we have 0 < 2mn 1 and thus,|2mn 1|< 1.So, we get |xn xm| < 2m ifn m N. Since mN, wehave 2m 2N and thus we get,

    |xn xm|< 2m 2N 1 =,

    where the last inequlaity follows from equation 1 and this isvalid for n m N. This is what we set out to prove andthus the sequence {xn}is a CS.

    (3) For any natural number n, we have 2n2 < 2n2 + 1. Thus by

    exercise (5), we can choose a rational numberynsuch that 2n

    2

    0, easy to see that there exists an N N such that

    for all n N, we have 0 < n2 < . Ifn m N, then wehave,

    |xn xm|< 2 +m2 2 =m2 <

    (4) Let

    xn= 1 +1

    2+

    1

    3+ +

    1

    nThen {xn} is not a CS. This is left as a not too easy exercise.

    Or may be look it up in your calculus text.5.2. Construction of Real Numbers. Next let Sbe the set of allCauchy Sequences in Q. We put a relation on Sas follows: {xn} {yn}, if given any 0 < Q, there exists an N N such that for alln, m N, we have|xn ym|< .

    This is indeed an equivalence relation. Reflexivity is just the fact thatthe sequences are Cauchy. Symmetry is obvious since|x y|= |y x|.Transitivity follows from triangle inequality (see Exercise 5).

  • 7/25/2019 Constructia multimilor de numere.pdf

    21/31

    CONSTRUCTION OF NUMBER SYSTEMS 21

    Thus we consider the set Ras the set of equivalence classes and callit the real numbers.

    Before we introduce the operations on R, let us prove a few thingsabout CS.

    Lemma 5.1. Let{xn} be a CS. Then there exists a rational numberM Q, such that |xn|< M for alln. That is to say, the sequence isbounded.

    Proof. Pick = 1. So we have an N N satisfying the properties ofthe definition of a CS. Let

    M= max{|x1|, |x2|, . . . , |xN1|, |xN|} + 1.

    By choice, |xn| < M if n N. Ifn > N, then by choice, we have,|xn xN| < 1 and then using triangle inequality (see Exercise 5), weare done.

    |xn|= |xn xN+xN| |xn xN| + |xN|< 1 + |xN| M

    As usual we define the operations as follows. If A = [{xn}] andB = [{yn}], define A B = [{xn+yn}] and A B = [{xnyn}]. Let uscheck that these make sense.

    Lemma 5.2. If {xn} and {yn} are CS, then so are {xn +yn} and{xnyn}.

    Proof. Given , we can find N1, N2 Nsuch that for all n, m N1 wehave|xn xm| < /2 and for all p.qN2, yp yq|< /2. TakeN =max{N1, N2}and use the triangle inequality to show that{xn+ yn}isCauchy.

    For the multiplication, we use lemma 5.1 and thus there existsM1, M2 Q such that |xn| < M1 for all n and |yn| < M2 for all n. Clearly,we may replace M1, M2 by M = max{M1, M2}. Given > 0, con-sider = /2M > 0. As before, there exists N1, N2 such that for alln, m N1, we have |xn xm| < etc. Again we may repalce N1, N2byN= max{N1, N2}. Thus we get,

    |xnyn xmym| = |(xn xm)yn+xm(yn ym)|

    |(xn xm)yn| + |xm(yn ym)|

    by triangle inequality. Ifn, m N, this in turn gives

    |xn xm||yn| + |xm||yn ym|< M+M =

    proving that our sequence is Cauchy.

  • 7/25/2019 Constructia multimilor de numere.pdf

    22/31

    22 N. MOHAN KUMAR

    Now, as usual, I will leave it to you to check that this definition ofaddition and multiplication are well defined. (Please try to check this

    it is a good exercise). I will check that addition is well defined below,just for illustration.

    Lemma 5.3. Addition of real numbers as defined above is well defined.

    Proof. Our definition was if A = [{xn}] and B = [{yn}], two realnumbers, thenA B = [{xn+yn}] and we have checked in the previouslemma that {xn+yn} is a CS. IfA= [{tn}] andB = [{un}], thenA Bis defined as [{tn+un}]. So, we must check that [{xn+yn}] = [{tn+un}].That is {xn+yn} {tn+un}. So, we must check that given >0 thereexists an N N such that for all n, m N,|xn+yn tm um|< .

    Since [{xn}] = [{tn}], by our definition {xn} {tn} and hence wecan find anN1 N so that for alln, mN1,|xntm|< /2. Similarlywe can find an N2 N so that for all n, m N2,|yn um|< /2. LetN= max{N1, N2}and then for any n, mN,

    |xn+yn tm um| |xn tm| + |yn um|<

    2+

    2=,

    the middle inequlity being the triangle inequality. This proves whatwe set out to prove.

    We also have a map f : Q R, sending a Q to the equivalenceclass of the CS, xn = a for all n(That this is indeed a CS was checked

    in Exercise 6). The functionf is one-one and thus we can identify Qas a subset ofR, f(a+ b) = f(a) f(b) and f(ab) = f(a) f(b).Thus now, we may drop our complicated notation and write the usualsymbols for addition and multiplication. Also, we can check all thestandard properties of this operation. We also define an ordering on Ras follows. If{xn} and {yn} are CS, and A= [{xn}] and B = [{yn}],then A < B, if there exists an > 0, rational number and an N Nsuch that for all n, m N, ym xn > . Again make sure that thisis well defined. If we define A B as usual, by saying that A < B orA= B , then one can easily check the following. A= {xn} B ={yn}if and only if foranypositive rational number, there exists an N such

    that for all n, mN, yn xm> .

    Exercise 7. Show that if{xn} is CS of rational numbers and {yn} isa subsequence of{xn} (which I have noted also must be a CS), thenshow that{xn} {yn}.

    5.3. Supremum and Infimum. Now we have all the machinery re-quired to prove the following important properties of the real numbers.The proofs, while elementary, are fairly subtle. You may try it for fun.

  • 7/25/2019 Constructia multimilor de numere.pdf

    23/31

    CONSTRUCTION OF NUMBER SYSTEMS 23

    If you do not succed, do not be discouraged. Again, as a warm upexercise, let us prove an easy lemma.

    Lemma 5.4. IfA < B are two real numbers, there is a rational numberq, such thatA < q < B. Remember that a rational number q as anelement ofR is just the equivalence class of the Cauchy sequence withall terms equal to q.

    Proof. Write A = [{xn}] and B = [{yn}]. Then by definition,A < Bmeans, there exists a positive rational number and an N1 N suchthat for alln, m N1,yn xm> . Since{xn}is a CS, there exists anN2 so that for all n, m N2, we have|xn xm|< /2. Similarly, thereexists N3 N so that for all n, m N3, |yn ym|< /2. If we choose

    N = max{N1, N2, N3}, then for all n, m N, all the above threeinequlaities hold. Now, let q = (xN+yN)/2. I claim, this rationalnumber is between A and B. We will show that q < B, and theinequalityA < qwill be similar.

    For n N, we should compute yn q.

    yn q=yn xN+yN

    2

    =yn xN

    2 +

    yn yN2

    Since n, NNN1, we have yn xN> . On the other hand, sincen, NNN3, we have |yn yN|< /2. This implies by lemma 2.7,yn yN>/2. Substituting these in the above, we get,

    yn q >

    2

    4=

    4

    This shows that q < B. Similarly one shows that A < q.

    Definition7. LetS R anda R. Thena is called a lower bound forS ifa s for all s S. Similarly an element b R is called an upperbound for S ifs b for all s S.

    Now, we prove the most important property of real numbers, fromwhich all the other subtle properties can be deduced. The proof is long

    and so take your time mulling over the steps.

    Theorem 5.1. LetS R be a non-empty subset and assume that ithas a lower bound M. Then there exists a real number (called theinfimum ofS) such that for anysS, s and ifx R is such thats x for alls S, then x.

    Proof. First, notice that we may assume the M that we have can beassumed to be rational, by choosing a smaller number by the previous

  • 7/25/2019 Constructia multimilor de numere.pdf

    24/31

    24 N. MOHAN KUMAR

    lemma. Our aim is to construct as in the theorem and by now weshould have the feeling that in general it is going to be a real number,

    but not a rational number. Thus to get there, we must construct anapproriate Cauchy sequence, which will be a real number using ourrelation. Let us during the proof, call a numbera R a lower boundfor S ifa s for all s S. So M is a lower bound. Now pick anys S. (This is where we use the fact that Sis not empty). Again, easyto see that we can pick a rational numberN > s. Letq= N M Q.Call M1 = M. Consider the rational number M+ (q/2). Then thereare two possibilities. Either this number is a lower bound for Sor not.If it is, call M2 = M+ (q/2). If it is not call M2 = M1. Let us see whatwe have.

    By choice,M2is still a lower bound for S,M1 M2,M2 M1 q/2and there exists ans Ssuch that s M2< q/2.

    Now we repeat the process. That is consider M2 +(q/4). Then againthere are two possibilities. Either it is a lower bound for S or not. Ifit is call M3 = M2+ (q/4) or else call M3=M2. Again notice that M3is a lower bound for S, M2 M3, M3 M2 q/4 and there exists ans S with s M3 < q/4. We continue this process by replacingq/4with q/8, q/16 etc. to get a sequence{Mn}.

    Next we check that this is indeed a Cauchy sequence and = [{Mn}]is an infimum forS. Let us repeat the basic properties of this sequenceof rational numbers.

    Mnis a lower bound for Sn N

    M1 M2 Mn Mn+1

    Mn+1 Mn q

    2n n N (2)

    sn Ssuch that sn Mn< q

    2n1, n N

    If one wants to be very precise, this is how the above should bephrased. We would like to construct recursively Mn for n N satisfy-ing the above properties. We are given a lower bound Mwhich we call

    M1. SinceS=, pick an elements Sand letNbe a rational numbersuch thatN > s. Letq= N Ma positive rational number. Then weconstruct M2 as described above, satisfying the properties in equation2 for n = 1, 2. So assume that we have constructedM1, M2, . . . , M nsatisfying the above properties. We wish to construct an Mn+1 satis-fying the above. So, we considerMn+

    q

    2n. If this number is a lower

    bound forS, we call thisMn+1. Otherwise we let Mn+1 to be the sameas Mn. So, by choice, we still have Mn+1 a lower bound for Sand we

  • 7/25/2019 Constructia multimilor de numere.pdf

    25/31

    CONSTRUCTION OF NUMBER SYSTEMS 25

    also have Mn Mn+1. Since Mn+1 Mn = 0 or q/2n, we also have

    Mn+1 Mn q/2n. So, we only need to verify the last requirement.

    For this again we look at the two cases when Mn+1 = Mn+ q2n orMn. In the first case, we take sn+1=sn. Then

    sn+1 Mn+1=sn Mn q

    2n 0, choose an N N so that q/2N1 < . This can be doneby lemma 2.6. Ifn m N, by equation 3, we get,

    |Mn Mm|< q

    2m1

    q

    2N1 < .

    This proves that {Mn} is a Cauchy sequence and so = [{Mn}] is areal number.

    Next, we check that is a lower bound for S. For this, lets S.and let > 0 be given. Then we may choose an N1 N so that

    q/2

    N11

    < /2 as before. Since MN1 is lower bound for S, we haveMN1 s. If we write s = [{un}] for a Cauchy sequence {un}, thereexists an N2 N so that for all n N2, un MN1 > /2, bydefinition of inequality discussed earlier. Now, letN= max{N1, N2}.Ifn, m N, we get, using equation 3,

    un Mm= un MN1+ MN1 Mm

    >

    2

    q

    2N11 >.

  • 7/25/2019 Constructia multimilor de numere.pdf

    26/31

    26 N. MOHAN KUMAR

    This proves that s.Finally we check that is an infimum for S. So, letx be a lower

    bound forS. We must show thatx . We prove this by contradiction.If this is not true, then x > and let us write x = [{xn}] as usual. So,there exists an >0 and N1 N so that for all n, m N1,

    xn Mm> . (4)

    Choose as before anN2so thatq/2N21 < /3. Then by equation 2, we

    have ans Sso that s MN2 < q/2N21, /3. Writing thiss = [{un}],

    there exists an N3 N so that for all n N3, un MN2 /3< /3.We rewrite this as,

    MN2 un>2

    3 (5)

    Now, letN= max{N1, N2, N3}. Then for alln, m N, we have, usingequations 2, 4 and 5,

    xn um = (xn MN) + (MN MN2) + (MN2 um)

    > + 0 2

    3 =

    3.

    Thus by definition, we get that x > s. This is a contradiction, since xwas a lower bound and hence x s for all sS.

    An identical argument can be used to prove the following,

    Theorem 5.2. LetS Rbe a non-empty subset and assume it has anupper bound. Then there exists a real number (called the supremumofS) such that for anys S, s and ifx R is such thats xfor allsS, thenx.

    Now, I repeat the properties of infimum and supremum explicitly, sothat we can use it again. These properties are easy, but the existenceas proved above is not.

    Lemma 5.5. LetSbe a non-empty set bounded below and let be its

    infimum. Then is a lower bound forS. Further, given any positivenumber, there exists ansSsuch that s < +.Similarly, ifS is non-empty set bounded above, then its supremum

    is an upper bound forS. Further given any positive number thereexists ans Sso that < s .

    Proof. The proof is easy. We already know that the infimum is a lowerbound. Now, assume that we are given > 0. Then by the propertyof infimum, + can not be a lower bound for S. But this means

  • 7/25/2019 Constructia multimilor de numere.pdf

    27/31

    CONSTRUCTION OF NUMBER SYSTEMS 27

    precisely that there is an s Swiths < +. The proof for supremumis identical.

    The phrasegreatest lower bound(glb for short) is used interchageablywith infimum and least upper bound(lub for short) for supremum.

    Next we define Cauchy Sequences exactly as before, but with realnumbers instead of rational numbers.

    Definition 8. A sequence of real numbers {An} is a CS, if for anypositive real number there exists anN N so that for all n, m N,|An Am|< .

    Of course, we could have defined a CS of real numbers with arational number.

    Definition 9. A sequence of real numbers {An} is a CS, if for anypositive rational number there exists anN Nso that for all n, mN,|An Am|< .

    Lemma 5.6. The two defintions above are equivalent. That is, a se-quence{An} of real numbers is a CS in the first definition if and onlyif it is so in the second definition.

    The proof is an easy application of lemma 5.4.

    Theorem 5.3. Let{xn} be a Cauchy sequence of real numbers. Thenthere exits a unique real number x such that given any > 0, realnumber, there exists anN N, such that for alln N, |xn x|< .

    The above theorem states that if we repeated the construction ofreals from rationals, then we get nothing new. This is usually termedas the completeness of the real numbers.

    Proof. We first look at non-empty sets, Si for i = 0, 1, . . . as follows.LetS0 ={x1, . . . , xn, . . .},S1 = {x2, x3, . . . , xn, . . .}etc. These are setsand not sequences (though they look like sequences). So, Sn would bethe set of elements of the sequence starting from xn+1. These are all

    non-empty and as we have seen in lemma 5.1, these are bounded, since{xn}is a CS. Thus by theorem 5.1, we have n the infimum ofSn.

    First notice that n n+1 for all n. This is because, since n is alower bound for the set Sn and Sn+1 Sn, it is clearly a lower boundfor Sn+1 and thus by property of infimum, we must have n n+1.Now, since all the s are bounded above, since{xn} is CS, we have asupremum for the non-empty set, {0, . . . , n, . . .}. Let this supremumbe x. I claim that this xhas the property stated in the theorem.

  • 7/25/2019 Constructia multimilor de numere.pdf

    28/31

    28 N. MOHAN KUMAR

    So, assume that we are given an >0 and let =/3. Then thereexists an N1 N so that for all n, m N1,

    |xn xm|< . (6)

    Since x is the supremum of the set {n}, by lemma 5.5, there exists anelement sayN2 so that, x < N2 x. Sincen n+1 for all n, wemay replace N1, N2 byN= max{N1, N2}. Thus, we have

    x < Nx. (7)

    Finally, since N is the infimum of the set SN, by lemma 5.5 again,there exists an element xl SNso that

    Nxl < N+ (8)

    Notice that since xl SN, l > N. Putting these three equationstogether, we get, for n N,

    |x xn|= |x N+N xl+xl xn|

    |x N| + |N xl| + |xl xn|

    < ++=

    Now, we only need to prove that this x is unique. I leave it as anexercise.

    Definition 10. If{xn} is a Cauchy sequence of real numbers and x is

    the unique real number we found in the above theorem, we call x thelimit of the sequence{xn} and write x= lim xn. For a set S, if it hasan infimum, we denote it by infSand similarly, if it has a supremumdenote it by sup S.

    Exercise 8. (1) Let x1 x2 x3 be a sequence (of realnumbers) which is bounded above. Show that{xn}is a CS andlim xn= sup{x1, x2, x3, . . .}.

    (2) Let {xn} be a CS and assume thatmis a lower bound for the set{xn} andMan upper bound. Then show thatm lim xn M.

    Theorem 5.4. LetSbe an infinite bounded set. That is, S is infiniteand there exists an M > 0 such that for all s S, |s| M. Thenthere exists an x R such that, for any > 0, there are infinitelymany elementss Ssuch that|x s|< .

    The proof is on similar lines as above and I will not prove it.By now, it should be clear to you, that while the arguments are not

    difficult, they can be rather tedious. These arguments repeat them-selves in several guises.

  • 7/25/2019 Constructia multimilor de numere.pdf

    29/31

    CONSTRUCTION OF NUMBER SYSTEMS 29

    6. Continuous functions

    In this section we study continuous functions from R to R. Youshould do these for functions defined in an open interval, but I will notgo into it in any detail since it is mostly routine. We start with thedefinition of a continuous function at a point x R.

    Definition 11. A function f : R R is called continuous at a pointx R if for any CS, {xn}, with lim xn = x, the sequence {f(xn)}is a CS. A function is continuous on R (or any open interval) if it iscontinuous at every point ofR (respectively, at every point of the openinterval).

    As usual, we will write [a, b] for a < b, the closed interval, which is

    the set of allxR

    such thata x b. Similarly, open and half-closedintervals can be defined.Before we give the usual examples of continuous functions, let me

    prove some easy lemmas.

    Lemma 6.1. Iff , gare continuous functions onR, so isf+ gandf g,where(f+g)(x) =f(x) +g(x) and(f g)(x) =f(x)g(x) for allx R.

    Proof is just an application of lemma 5.2.

    Lemma 6.2. Iff is continuous atx and{xn}is any CS withlim xn=x, thenlim f(xn) =f(x).

    Proof. Consider a new sequence {yn}defined as follows. For n = 2m

    1, define yn = xm and for n = 2m define yn = x. It is easy to checkthat then {yn} is a CS and lim yn = x. So, by continuity, {f(yn)} isa CS. Let y = lim f(yn). So, given any > 0, there exists an N suchthat for n N, we have |f(yn) y | < . But, if n N and n iseven, since yn = x, we get |f(x) y| < . But, since was arbitrary,this can happen only ify = f(x). Now, taking 2m 1 = n N, onehas yn = xm and so we get |f(xm) f(x)| < , which implies thatlim f(xn) =f(x).

    Example 2. (1) The identity function Id : R R is continuous.

    That is, the function Id(x) =x is continuous.(2) By the lemma above, we see that the function f(x) = xn is

    continuous for any n N.(3) Polynomial functions are continuous. These are functions of the

    form, f(x) =a0xn + a1x

    n1 + + an, wheren N andai R.

    Next let me prove a fundamental theorem about continuous func-tions, which is frequently used as the definition, often called the -definition of continuity.

  • 7/25/2019 Constructia multimilor de numere.pdf

    30/31

    30 N. MOHAN KUMAR

    Theorem 6.1. Let f be a function (from R or an open interval toR). Thenf is continuous at a pointx if and only if, given any >0,

    there exists a >0 such that for any t such that|t x|< , we have|f(t) f(x)|< .

    Proof. First let us assume that fis continuous. The proof is by contra-diction. So, assume that we are give an >0 and assume that there isno >0 satisfying the above condition. Then for any n N, there ex-ists anxnsuch that |xnx|< 1/nand |f(xn)f(x)| . Consider thesequence {xn}. It is immediate that {xn} is a CS and lim xn=x. Sincefis continuous, we must have {f(xn)} a CS and lim f(xn) =f(x). But,this means that for all n >> 0, |f(xn) f(x)| < , which contradictsthe previous inequality.

    To prove the converse, assume we are given a CS{xn}with lim xn=x. Given an >0, we have a >0 so that for all t with |t x| < ,|f(t) f(x)|< /2. Since lim xn = x, there exists an Nso that for alln N,|xn x|< . So, ifn, m N, we get,

    |f(xn) f(xm)|= |f(xn) f(x) +f(x) f(xm)|

    |f(xn) f(x)| + |f(xm) f(x)|

    <

    2+

    2=

    This shows that{f(xn)} is a CS, proving continuity.

    We next prove the last theorem for this topic, used often by all ofyou in your calculus classes.

    Theorem 6.2 (Intermediate Value Theorem). Let f be a continuosfunction (onR or in the closed interval[a, b]) wherea < b. Then givenany real number u between f(a) and f(b), there exists a real numbera c b such thatf(c) =u.

    Proof. Iff(a) =f(b), thenu = f(a) and there is nothing to prove. So,we may assume f(a)=f(b). So, we will assume that f(a)< f(b), thecase f(a)> f(b) being similar. We may also assume thatf(a) < u u. Notice that c > a, since otherwise, c = a and

    then f(c) = f(a) < u. Let 0 < = c a. Then for all n >> 0,natural numbers we have a c 1/n < c. Since c was the supremumof the set S, there must exist an xn S with c 1/n < xn c. Itis easy to see that {xn} is a CS and lim xn =c. So, by continuity wehave lim f(xn) = f(c). But, sincef(xn) u becuase xn S, we seethat uis an upper bound for the set {f(xn)}and hence by exercise 8,f(c) u. This is a contradiction.

    Next we show that the assumption f(c) < u also leads to a contra-diction and then we would have proved the result. So, assume thatf(c) < u. Choose an > 0 such that f(c) + < u. (For example,you could choose = (u f(c))/2). Then there exists a > 0, bycontinuity off such that for all t with |t c| < , |f(t) f(c)| < .We will then show that, if tc+/2, then f(t) u. Ift < c, thereexists an x Ssuch that t < x c and we know that for any such t,f(t) u by defintion of our set S. Ift= c, this is our assumption. Ifc < t c +/2, we know that |f(t)f(c)|< and thusf(t)f(c)< .This meansf(t)< f(c) + < u. Thus, we see that c + /2 Sby ourdefintion of the set S. But, thenc < c+/2 can not be a supremumfor S, since it is not an upper bound for S. This contradcition provesthe theorem.