• Tidak ada hasil yang ditemukan

Basic properties of the integers

N/A
N/A
Protected

Academic year: 2024

Membagikan "Basic properties of the integers"

Copied!
14
0
0

Teks penuh

(1)

1

Basic properties of the integers

This chapter discusses some of the basic properties of the integers, including the notions of divisibility and primality, unique factorization into primes, greatest com- mon divisors, and least common multiples.

1.1 Divisibility and primality A central concept in number theory isdivisibility.

Consider the integersZ= {. . . ,−2,−1, 0, 1, 2, . . .}. Fora,b∈Z, we say thata dividesbifaz=bfor somez∈Z. Ifadividesb, we writea|b, and we may say thatais adivisorofb, or thatbis amultipleofa, or thatbisdivisible bya. Ifa does not divideb, then we writea-b.

We first state some simple facts about divisibility:

Theorem 1.1. For all a,b,c∈Z, we have (i) a|a,1|a, and a|0;

(ii) 0|aif and only if a=0;

(iii) a|bif and only if −a|bif and only if a| −b;

(iv) a|banda|cimpliesa|(b+c);

(v) a|bandb|cimplies a|c.

Proof. These properties can be easily derived from the definition of divisibility, using elementary algebraic properties of the integers. For example,a | abecause we can writea·1=a; 1|abecause we can write 1·a=a;a|0 because we can writea·0=0. We leave it as an easy exercise for the reader to verify the remaining properties. 2

We make a simple observation: ifa | bandb 6= 0, then 1 ≤ |a| ≤ |b|. Indeed, ifaz = b 6= 0 for some integerz, thena 6= 0 andz 6= 0; it follows that|a| ≥ 1,

|z| ≥1, and so|a| ≤ |a||z|=|b|.

1

(2)

Theorem 1.2. For all a,b∈Z, we havea| band b|aif and only if ab. In particular, for everya∈Z, we havea|1if and only if a=±1.

Proof. Clearly, ifa = ±b, thena | bandb | a. So let us assume that a | band b|a, and prove thatab. If either ofaorbare zero, then the other must be zero as well. So assume that neither is zero. By the above observation,a | bimplies

|a| ≤ |b|, andb|aimplies|b| ≤ |a|; thus,|a|=|b|, and soab. That proves the first statement. The second statement follows from the first by settingb:=1, and noting that 1|a. 2

The product of any two non-zero integers is again non-zero. This implies the usualcancellation law: ifa,b, andcare integers such thata6=0 andab=ac, then we must haveb= c; indeed,ab =acimpliesa(bc) = 0, and soa 6= 0 implies bc=0, and henceb=c.

Primes and composites. Letnbe a positive integer. Trivially, 1 and ndividen.

Ifn > 1 and no other positive integers besides 1 andndividen, then we saynis prime. Ifn >1 butnis not prime, then we say thatniscomposite. The number 1 is not considered to be either prime or composite. Evidently,nis composite if and only ifn= abfor some integersa,bwith 1< a < nand 1< b < n. The first few primes are

2, 3, 5, 7, 11, 13, 17, . . . .

While it is possible to extend the definition of prime and composite to negative integers, we shall not do so in this text:whenever we speak of a prime or composite number, we mean a positive integer.

A basic fact is that every non-zero integer can be expressed as a signed product of primes in an essentially unique way. More precisely:

Theorem 1.3 (Fundamental theorem of arithmetic). Every non-zero integer n can be expressed as

npe11· · ·perr,

wherep1, . . . ,prare distinct primes and e1, . . . ,erare positive integers. Moreover, this expression is unique, up to a reordering of the primes.

Note that ifn = ±1 in the above theorem, thenr = 0, and the product of zero terms is interpreted (as usual) as 1.

The theorem intuitively says that the primes act as the “building blocks” out of which all non-zero integers can be formed by multiplication (and negation).

The reader may be so familiar with this fact that he may feel it is somehow “self evident,” requiring no proof; however, this feeling is simply a delusion, and most

(3)

1.1 Divisibility and primality 3 of the rest of this section and the next are devoted to developing a proof of this theorem. We shall give a quite leisurely proof, introducing a number of other very important tools and concepts along the way that will be useful later.

To prove Theorem 1.3, we may clearly assume thatnis positive, since otherwise, we may multiplynby−1 and reduce to the case wherenis positive.

The proof of the existence part of Theorem 1.3 is easy. This amounts to showing that every positive integer n can be expressed as a product (possibly empty) of primes. We may prove this by induction onn. Ifn = 1, the statement is true, as n is the product of zero primes. Now letn > 1, and assume that every positive integer smaller thann can be expressed as a product of primes. If nis a prime, then the statement is true, asnis the product of one prime. Assume, then, thatn is composite, so that there exista,b ∈Zwith 1< a < n, 1< b < n, andn= ab.

By the induction hypothesis, bothaandbcan be expressed as a product of primes, and so the same holds forn.

The uniqueness part of Theorem 1.3 is the hard part. An essential ingredient in this proof is the following:

Theorem 1.4 (Division with remainder property). Let a,b ∈ Z with b > 0.

Then there exist uniqueq,r∈Zsuch thata=bq+rand 0≤r < b.

Proof. Consider the setSof non-negative integers of the formabtwitht ∈Z. This set is clearly non-empty; indeed, ifa≥0, sett:= 0, and ifa <0, sett:= a.

Since every non-empty set of non-negative integers contains a minimum, we define rto be the smallest element ofS. By definition,ris of the formr = abq for someq∈Z, andr≥0. Also, we must haver < b, since otherwise,rbwould be an element ofSsmaller thanr, contradicting the minimality ofr; indeed, ifrb, then we would have 0≤rb=ab(q+1).

That proves the existence ofrandq. For uniqueness, suppose thata = bq+r anda = bq0+r0, where 0 ≤ r < band 0 ≤ r0 < b. Then subtracting these two equations and rearranging terms, we obtain

r0r=b(qq0).

Thus, r0r is a multiple of b; however, 0 ≤ r < b and 0 ≤ r0 < b implies

|r0r|< b; therefore, the only possibility isr0r =0. Moreover, 0 =b(qq0) andb6=0 impliesqq0=0. 2

Theorem 1.4 can be visualized as follows:

0 r b 2b 3b a 4b

(4)

Starting witha, we subtract (or add, ifais negative) the valuebuntil we end up with a number in the interval [0,b).

Floors and ceilings. Let us briefly recall the usual floorand ceiling functions, denotedb·candd·e, respectively. These are functions fromR(the real numbers) toZ. Forx∈R,bxcis the greatest integermx; equivalently,bxcis the unique integermsuch that mx < m+1, or put another way, such thatx = m+εfor someε ∈[0, 1). Also,dxeis the smallest integermx; equivalently,dxeis the unique integermsuch thatm−1< xm, or put another way, such thatx=mε for someε∈[0, 1).

The mod operator.Now leta,b∈Zwithb >0. Ifqandrare the unique integers from Theorem 1.4 that satisfya=bq+rand 0≤r < b, we define

amodb:=r;

that is,amodbdenotes the remainder in dividingabyb. It is clear thatb | aif and only ifamodb= 0. Dividing both sides of the equationa= bq+rbyb, we obtaina/b=q+r/b. Sinceq ∈Zandr/b∈[0, 1), we see thatq=ba/bc. Thus,

(amodb)=abba/bc.

One can use this equation to extend the definition ofamodbto all integersaand b, withb6=0; that is, forb <0, we simply defineamodbto beabba/bc.

Theorem 1.4 may be generalized so that when dividing an integeraby a positive integer b, the remainder is placed in an interval other than [0,b). Let x be any real number, and consider the interval [x,x+b). As the reader may easily verify, this interval contains preciselybintegers, namely,dxe, . . . ,dxe+b−1. Applying Theorem 1.4 witha− dxein place ofa, we obtain:

Theorem 1.5. Let a,b ∈ Zwith b > 0, and let x ∈ R. Then there exist unique q,r∈Zsuch thata=bq+rand r∈[x,x+b).

EXERCISE 1.1. Leta,b,d∈Zwithd6=0. Show thata|bif and only ifda|db.

EXERCISE 1.2. Letn be a composite integer. Show that there exists a prime p dividingn, withpn1/2.

EXERCISE 1.3. Letmbe a positive integer. Show that for every real numberx≥1, the number of multiples ofmin the interval [1,x] isbx/mc; in particular, for every integern≥1, the number of multiples ofmamong 1, . . . ,nisbn/mc.

EXERCISE 1.4. Letx∈R. Show that 2bxc ≤ b2xc ≤2bxc+1.

(5)

1.2 Ideals and greatest common divisors 5 EXERCISE 1.5. Letx∈Randn∈Zwithn >0. Show thatbbxc/nc=bx/nc; in particular,bba/bc/cc=ba/bccfor all positive integersa,b,c.

EXERCISE 1.6. Leta,b∈Zwithb <0. Show that (amodb) ∈(b, 0].

EXERCISE1.7. Show that Theorem 1.5 also holds for the interval (x,x+b]. Does it hold in general for the intervals [x,x+b] or (x,x+b)?

1.2 Ideals and greatest common divisors

To carry on with the proof of Theorem 1.3, we introduce the notion of anideal of Z, which is a non-empty set of integers that is closed under addition, and closed under multiplication by an arbitrary integer. That is, a non-empty setI ⊆Zis an ideal if and only if for alla,bIand allz∈Z, we have

a+bI and azI.

Besides its utility in proving Theorem 1.3, the notion of an ideal is quite useful in a number of contexts, which will be explored later.

It is easy to see that every idealI contains 0: sinceaI for some integer a, we have 0 = a·0 ∈I. Also, note that if an idealI contains an integera, it also contains−a, since−a = a·(−1) ∈I. Thus, if an ideal containsaandb, it also containsab. It is clear that{0}andZare ideals. Moreover, an idealI is equal toZif and only if 1∈I; to see this, note that 1 ∈Iimplies that for everyz∈Z, we havez= 1·zI, and henceI = Z; conversely, ifI = Z, then in particular, 1∈I.

Fora∈Z, defineaZ:={az:z∈Z}; that is,aZis the set of all multiples ofa.

Ifa=0, then clearlyaZ={0}; otherwise,aZconsists of the distinct integers . . . ,−3a,−2a,−a, 0,a, 2a, 3a, . . . .

It is easy to see that aZ is an ideal: for allaz,az0aZ andz00 ∈ Z, we have az+az0 = a(z+z0) ∈ aZ and (az)z00 = a(zz00) ∈ aZ. The idealaZis called theideal generated bya, and an ideal of the formaZfor somea ∈Zis called a principal ideal.

Observe that for all a,b ∈ Z, we have baZ if and only if a | b. Also observe that for every ideal I, we havebI if and only ifbZ ⊆ I. Both of these observations are simple consequences of the definitions, as the reader may verify. Combining these two observations, we see thatbZ⊆aZif and only ifa|b.

SupposeI1andI2are ideals. Then it is not hard to see that the set I1+I2:={a1+a2 :a1I1,a2I2}

(6)

is also an ideal. Indeed, supposea1+a2I1+I2andb1+b2I1+I2. Then we have (a1+a2)+(b1+b2)=(a1+b1)+(a2+b2)∈I1+I2, and for everyz∈Z, we have (a1+a2)z=a1z+a2zI1+I2.

Example 1.1. Consider the principal ideal 3Z. This consists of all multiples of 3;

that is, 3Z={. . . ,−9,−6,−3, 0, 3, 6, 9, . . .}. 2

Example 1.2. Consider the ideal 3Z+5Z. This ideal contains 3·2+5·(−1)=1.

Since it contains 1, it contains all integers; that is, 3Z+5Z=Z. 2

Example 1.3. Consider the ideal 4Z+6Z. This ideal contains 4·(−1)+6·1=2, and therefore, it contains all even integers. It does not contain any odd integers, since the sum of two even integers is again even. Thus, 4Z+6Z=2Z. 2

In the previous two examples, we defined an ideal that turned out upon closer inspection to be a principal ideal. This was no accident: the following theorem says that all ideals ofZare principal.

Theorem 1.6. Let I be an ideal of Z. Then there exists a unique non-negative integer dsuch that I=dZ.

Proof. We first prove the existence part of the theorem. IfI = {0}, thend = 0 does the job, so let us assume thatI 6= {0}. SinceIcontains non-zero integers, it must contain positive integers, since ifaI then so is−a. Letdbe the smallest positive integer inI. We want to show thatI=dZ.

We first show that IdZ. To this end, leta be any element inI. It suffices to show thatd | a. Using the division with remainder property, writea = dq+r, where 0≤r < d. Then by the closure properties of ideals, one sees thatr=adq is also an element of I, and by the minimality of the choice ofd, we must have r=0. Thus,d|a.

We have shown thatIdZ. The fact thatdZ ⊆ I follows from the fact that dI. Thus,I=dZ.

That proves the existence part of the theorem. For uniqueness, note that if dZ = eZfor some non-negative integer e, thend | e ande | d, from which it follows by Theorem 1.2 thatde; sincedandeare non-negative, we must have d=e. 2

Greatest common divisors. For a,b∈Z, we calld∈ Zacommon divisorofa andbifd|aandd|b; moreover, we call such adagreatest common divisorof aandbifdis non-negative and all other common divisors ofaandbdivided.

Theorem 1.7. For all a,b∈Z, there exists a unique greatest common divisor dof aand b, and moreover,aZ+bZ=dZ.

(7)

1.2 Ideals and greatest common divisors 7 Proof. We apply the previous theorem to the idealI :=aZ+bZ. Letd∈Zwith I =dZ, as in that theorem. We wish to show thatdis a greatest common divisor ofaandb. Note thata,b,dIanddis non-negative.

Since aI = dZ, we see that d | a; similarly,d | b. So we see that dis a common divisor ofaandb.

SincedI =aZ+bZ, there exists,t∈Zsuch thatas+bt=d. Now suppose a=a0d0andb=b0d0for somea0,b0,d0∈Z. Then the equationas+bt=dimplies thatd0(a0s+b0t)=d, which says thatd0 |d. Thus, any common divisord0ofaand bdividesd.

That proves thatdis a greatest common divisor ofaandb. For uniqueness, note that ife is a greatest common divisor ofa andb, thend | eande | d, and hence de; since bothdandeare non-negative by definition, we haved=e. 2

Fora,b∈Z, we write gcd(a,b) for the greatest common divisor ofaandb. We say thata,b∈Zarerelatively primeif gcd(a,b) =1, which is the same as saying that the only common divisors ofaandbare±1.

The following is essentially just a restatement of Theorem 1.7, but we state it here for emphasis:

Theorem 1.8. Leta,b,r∈Zand letd:=gcd(a,b). Then there exist s,t∈Zsuch that as+bt= rif and only if d| r. In particular,aand bare relatively prime if and only if there exist integerssandtsuch thatas+bt=1.

Proof. We have

as+bt=r for somes,t∈Z

⇐⇒ raZ+bZ

⇐⇒ rdZ (by Theorem 1.7)

⇐⇒ d|r.

That proves the first statement. The second statement follows from the first, setting r:=1. 2

Note that as we have defined it, gcd(0, 0) = 0. Also note that when at least one ofaorbare non-zero, gcd(a,b) may be characterized as thelargestpositive integer that divides bothaandb, and as thesmallestpositive integer that can be expressed asas+btfor integerssandt.

Theorem 1.9. Let a,b,c∈Zsuch that c|aband gcd(a,c)=1. Thenc|b.

Proof. Suppose that c | ab and gcd(a,c) = 1. Then since gcd(a,c) = 1, by Theorem 1.8 we haveas+ct= 1 for somes,t∈Z. Multiplying this equation by

(8)

b, we obtain

abs+cbt=b. (1.1)

Sincecdividesabby hypothesis, and sincecclearly dividescbt, it follows thatc divides the left-hand side of (1.1), and hence thatcdividesb. 2

Suppose thatpis a prime andais any integer. As the only divisors ofpare±1 and±p, we have

p|a =⇒ gcd(a,p)=p, and p-a =⇒ gcd(a,p)=1.

Combining this observation with the previous theorem, we have:

Theorem 1.10. Let pbe prime, and let a,b∈Z. Thenp|abimplies that p|aor p|b.

Proof. Assume thatp|ab. Ifp|a, we are done, so assume thatp-a. By the above observation, gcd(a,p)=1, and so by Theorem 1.9, we havep|b. 2

An obvious corollary to Theorem 1.10 is that ifa1, . . . ,ak are integers, and ifp is a prime that divides the producta1· · ·ak, thenp|aifor somei=1, . . . ,k. This is easily proved by induction onk. Fork =1, the statement is trivially true. Now letk >1, and assume that statement holds fork−1. Then by Theorem 1.10, either p|a1orp|a2· · ·ak; ifp|a1, we are done; otherwise, by induction,pdivides one ofa2, . . . ,ak.

Finishing the proof of Theorem 1.3.We are now in a position to prove the unique- ness part of Theorem 1.3, which we can state as follows: ifp1, . . . ,pr are primes (not necessarily distinct), andq1, . . . ,qsare primes (also not necessarily distinct), such that

p1· · ·pr =q1· · ·qs, (1.2) then (p1, . . . ,pr) is just a reordering of (q1, . . . ,qs). We may prove this by induction on r. Ifr = 0, we must haves = 0 and we are done. Now supposer > 0, and that the statement holds for r −1. Since r > 0, we clearly must have s > 0.

Also, asp1 obviously divides the left-hand side of (1.2), it must also divide the right-hand side of (1.2); that is, p1 | q1· · ·qs. It follows from (the corollary to) Theorem 1.10 thatp1 | qjfor somej = 1, . . . ,s, and moreover, sinceqjis prime, we must havep1 = qj. Thus, we may cancel p1 from the left-hand side of (1.2) andqj from the right-hand side of (1.2), and the statement now follows from the induction hypothesis. That proves the uniqueness part of Theorem 1.3.

(9)

1.2 Ideals and greatest common divisors 9 EXERCISE 1.8. LetIbe a non-empty set of integers that is closed under addition (i.e.,a+bIfor alla,bI). Show thatIis an ideal if and only if−aIfor all aI.

EXERCISE 1.9. Show that for all integersa,b,c, we have:

(a) gcd(a,b)=gcd(b,a);

(b) gcd(a,b)=|a| ⇐⇒ a|b;

(c) gcd(a, 0)=gcd(a,a)=|a|and gcd(a, 1)=1;

(d) gcd(ca,cb)=|c|gcd(a,b).

EXERCISE 1.10. Show that for all integersa,bwithd:= gcd(a,b) 6=0, we have gcd(a/d,b/d) =1.

EXERCISE 1.11. Letnbe an integer. Show that ifa,bare relatively prime integers, each of which dividesn, thenabdividesn.

EXERCISE 1.12. Show that two integers are relatively prime if and only if there is no one prime that divides both of them.

EXERCISE 1.13. Leta,b1, . . . ,bk be integers. Show that gcd(a,b1· · ·bk) = 1 if and only if gcd(a,bi) =1 fori=1, . . . ,k.

EXERCISE 1.14. Letpbe a prime andkan integer, with 0< k < p. Show that the binomial coefficient

p k

= p!

k!(pk)!, which is an integer (see §A2), is divisible byp.

EXERCISE 1.15. An integer a is calledsquare-free if it is not divisible by the square of any integer greater than 1. Show that:

(a) a is square-free if and only ifa = ±p1· · ·pr, where thepi’s are distinct primes;

(b) every positive integerncan be expressed uniquely asn=ab2, whereaand bare positive integers, andais square-free.

EXERCISE 1.16. For each positive integerm, letIm denote{0, . . . ,m−1}. Let a,bbe positive integers, and consider the map

τ : Ib×IaIab

(s,t)7→(as+bt) modab.

Showτis a bijection if and only if gcd(a,b)=1.

(10)

EXERCISE 1.17. Let a,b,c be positive integers satisfying gcd(a,b) = 1 and c ≥ (a− 1)(b− 1). Show that there exist non-negative integers s,t such that c=as+bt.

EXERCISE 1.18. For each positive integer n, let Dn denote the set of positive divisors ofn. Letn1,n2be relatively prime, positive integers. Show that the sets Dn1 ×Dn2 and Dn1n2 are in one-to-one correspondence, via the map that sends (d1,d2)∈Dn1 ×Dn2 tod1d2.

1.3 Some consequences of unique factorization

The following theorem is a consequence of just the existence part of Theorem 1.3:

Theorem 1.11. There are infinitely many primes.

Proof. By way of contradiction, suppose that there were only finitely many primes;

call themp1, . . . ,pk. Then setM := Qk

i=1piandN :=M +1. Consider a prime p that divides N. There must be at least one such prime p, since N ≥ 2, and every positive integer can be written as a product of primes. Clearly, p cannot equal any of thepi’s, since if it did, thenpwould divideM, and hence also divide NM =1, which is impossible. Therefore, the primepis not amongp1, . . . ,pk, which contradicts our assumption that these are the only primes. 2

For each primep, we may define the functionνp, mapping non-zero integers to non-negative integers, as follows: for every integern6=0, ifn=pem, wherep-m, thenνp(n) :=e. We may then write the factorization ofninto primes as

n=±Y

p

pνp(n),

where the product is over all primes p; although syntactically this is an infinite product, all but finitely many of its terms are equal to 1, and so this expression makes sense.

Observe that ifaandbare non-zero integers, then

νp(a·b) =νp(a)+νp(b) for all primesp, (1.3) and

a|b ⇐⇒ νp(a)≤νp(b) for all primesp. (1.4) From this, it is clear that

gcd(a,b)=Y

p

pmin(νp(a),νp(b)).

(11)

1.3 Some consequences of unique factorization 11 Least common multiples. For a,b ∈ Z, acommon multiple of a andb is an integer msuch thata | mandb | m; moreover, such anmis the least common multipleofa andbifmis non-negative andmdivides all common multiples of a and b. It is easy to see that the least common multiple exists and is unique, and we denote the least common multiple ofaandbby lcm(a,b). Indeed, for all a,b∈Z, if eitheraorbare zero, the only common multiple ofaandbis 0, and so lcm(a,b)=0; otherwise, if neitheranorbare zero, we have

lcm(a,b) =Y

p

pmax(νp(a),νp(b)),

or equivalently, lcm(a,b) may be characterized as the smallest positive integer divisible by bothaandb.

It is convenient to extend the domain of definition of νp to include 0, defining νp(0) :=∞. If we interpret expressions involving “∞” appropriately (see Prelimi- naries), then for arbitrarya,b∈Z, both (1.3) and (1.4) hold, and in addition,

νp(gcd(a,b))=min(νp(a),νp(b)) and νp(lcm(a,b))=max(νp(a),νp(b)) for all primesp.

Generalizing gcd’s and lcm’s to many integers. It is easy to generalize the notions of greatest common divisor and least common multiple from two integers to many integers. Leta1, . . . ,ak be integers. We call d ∈ Z a common divisor ofa1, . . . ,ak if d | ai fori = 1, . . . ,k; moreover, we call such a dthe greatest common divisor of a1, . . . ,ak if d is non-negative and all other common divi- sors ofa1, . . . ,ak divided. The greatest common divisor ofa1, . . . ,ak is denoted gcd(a1, . . . ,ak) and is the unique non-negative integerdsatisfying

νp(d)=min(νp(a1), . . . ,νp(ak)) for all primesp.

Analogously, we call m ∈ Z a common multiple of a1, . . . ,ak if ai | m for all i=1, . . . ,k; moreover, such anmis called the least common multiple ofa1, . . . ,ak

if mdivides all common multiples ofa1, . . . ,ak. The least common multiple of a1, . . . ,ak is denoted lcm(a1, . . . ,ak) and is the unique non-negative integermsat- isfying

νp(m)=max(νp(a1), . . . ,νp(ak)) for all primesp.

Finally, we say that the family{ai}ki=1ispairwise relatively primeif for all indices i,jwithi6= j, we have gcd(ai,aj) =1. Certainly, if{ai}ki=1 is pairwise relatively prime, andk >1, then gcd(a1, . . . ,ak)=1; however, gcd(a1, . . . ,ak) =1 does not imply that{ai}ki=1is pairwise relatively prime.

(12)

Rational numbers. Consider the rational numbersQ= {a/b :a,b∈Z, b6= 0}.

Given any rational numbera/b, if we set d := gcd(a,b), and define the integers a0 := a/dandb0 :=b/d, then we havea/b= a0/b0 and gcd(a0,b0) = 1. More- over, if a1/b1 = a0/b0, then we havea1b0 = a0b1, and sob0 | a0b1; also, since gcd(a0,b0) =1, we see thatb0| b1; writingb1 =b0c, we see thata1=a0c. Thus, we can represent every rational number as a fraction inlowest terms, which means a fraction of the form a0/b0 wherea0 andb0 are relatively prime; moreover, the values of a0 andb0 are uniquely determined up to sign, and every other fraction that represents the same rational number is of the forma0c/b0c, for some non-zero integerc.

EXERCISE 1.19. Let n be an integer. Generalizing Exercise 1.11, show that if {ai}ki=1 is a pairwise relatively prime family of integers, where eachaidividesn, then their productQk

i=1aialso dividesn.

EXERCISE 1.20. Show that for all integersa,b,c, we have:

(a) lcm(a,b)=lcm(b,a);

(b) lcm(a,b)=|a| ⇐⇒ b|a;

(c) lcm(a,a) =lcm(a, 1)=|a|;

(d) lcm(ca,cb)=|c|lcm(a,b).

EXERCISE 1.21. Show that for all integersa,b, we have:

(a) gcd(a,b)·lcm(a,b) =|ab|;

(b) gcd(a,b)=1 =⇒ lcm(a,b) =|ab|.

EXERCISE 1.22. Leta1, . . . ,ak ∈Zwithk >1. Show that:

gcd(a1, . . . ,ak)=gcd(a1, gcd(a2, . . . ,ak))=gcd(gcd(a1, . . . ,ak−1),ak);

lcm(a1, . . . ,ak)=lcm(a1, lcm(a2, . . . ,ak))=lcm(lcm(a1, . . . ,ak−1),ak).

EXERCISE 1.23. Leta1, . . . ,ak ∈Zwithd := gcd(a1, . . . ,ak). Show thatdZ = a1Z+· · ·+akZ; in particular, there exist integersz1, . . . ,zk such thatd=a1z1+

· · ·+akzk.

EXERCISE 1.24. Show that if{ai}ki=1is a pairwise relatively prime family of inte- gers, then lcm(a1, . . . ,ak) =|a1· · ·ak|.

EXERCISE 1.25. Show that every non-zerox∈Qcan be expressed as xpe11· · ·perr,

where thepi’s are distinct primes and the ei’s are non-zero integers, and that this expression in unique up to a reordering of the primes.

(13)

1.3 Some consequences of unique factorization 13 EXERCISE 1.26. Letnandkbe positive integers, and suppose x ∈ Qsuch that xk =nfor somex ∈Q. Show thatx∈Z. In other words,√k

nis either an integer or is irrational.

EXERCISE 1.27. Show that gcd(a+b, lcm(a,b))=gcd(a,b) for alla,b∈Z.

EXERCISE 1.28. Show that for every positive integerk, there existkconsecutive composite integers. Thus, there are arbitrarily large gaps between primes.

EXERCISE1.29. Letpbe a prime. Show that for alla,b∈Z, we haveνp(a+b) ≥ min{νp(a),νp(b)}, andνp(a+b) =νp(a) ifνp(a)< νp(b).

EXERCISE 1.30. For a given primep, we may extend the domain of definition of νp fromZtoQ: for non-zero integersa,b, let us defineνp(a/b) := νp(a)−νp(b).

Show that:

(a) this definition of νp(a/b) is unambiguous, in the sense that it does not depend on the particular choice ofaandb;

(b) for allx,y∈Q, we haveνp(xy) =νp(x)+νp(y);

(c) for allx,y ∈Q, we haveνp(x+y) ≥ min{νp(x),νp(y)}, andνp(x+y) = νp(x) ifνp(x)< νp(y);

(d) for all non-zerox∈Q, we havex=±Q

ppνp(x), where the product is over all primes, and all but a finite number of terms in the product are equal to 1;

(e) for allx∈Q, we havex∈Zif and only ifνp(x)≥0 for all primesp.

EXERCISE 1.31. Letnbe a positive integer, and let 2k be the highest power of 2 in the setS:={1, . . . ,n}. Show that 2k does not divide any other element inS.

EXERCISE 1.32. Letn∈Zwithn >1. Show thatPn

i=11/iis not an integer.

EXERCISE1.33. Letnbe a positive integer, and letCndenote the number of pairs of integers (a,b) witha,b∈ {1, . . . ,n}and gcd(a,b) =1, and letFnbe the number ofdistinctrational numbersa/b, where 0≤a < bn.

(a) Show thatFn=(Cn+1)/2.

(b) Show thatCnn2/4. Hint: first show thatCnn2(1−P

d≥21/d2), and then show thatP

d≥21/d2≤3/4.

EXERCISE 1.34. This exercise develops a characterization of least common mul- tiples in terms of ideals.

(a) Arguing directly from the definition of an ideal, show that ifI andJ are ideals ofZ, then so isIJ.

(b) Let a,b ∈ Z, and consider the ideals I := aZ and J := bZ. By part

(14)

(a), we know that IJ is an ideal. By Theorem 1.6, we know that IJ = mZfor some uniquely determined non-negative integerm. Show thatm=lcm(a,b).

Referensi

Dokumen terkait

In this chapter, we describe the basic properties of spoken word production, outlining empirical data that demonstrate the properties of the processes resulting in speech and

Chapter 1 Chapter 2 Chapter 3 Chapter 4 Chapter 5 Chapter 6 Chapter 7 Appendix I Appendix II TABLE OF CONTENTS INTRODUCTION BASIC PRINCIPLES OF SHOCK WAVES IN SOLIDS SHOCK

On the Inverse of Bipartite Graphs with Unique Perfect Matchings and Reciprocal Eigenvalue Properties A thesis submitted in partial fulfilment of the requirements for the degree of

Based on understanding the surface properties of Al2O3, Chapter 4 shows how the number and properties of specific sites on Al2O3 affect the interaction between the supported active

2.8 Chapter Summary Chapter: 3-Theorizing and Framing the Study within the Context of Teacher Learning 3.1 Introduction 3.2 Re-examining Traditional Notions of Professional

Results and discussion This section discusses results obtained from the basic characterization of thin films such as microstructure properties of the materials, morphology, grain

Part Two consists of the studies on the properties and the the reliability of the oxide and the interface: pressure dependence of SiO2 growth kinetics Chapter III, impact of nitrogen

Chapter 2 The Thermal Properties of Iron-bearing Silicate Perovskite and the Implications for Lower Mantle Structures Abstract The high-temperature and -pressure equations of state