Course 2316 Sample Paper 1

Size: px
Start display at page:

Download "Course 2316 Sample Paper 1"

Transcription

1 Course 2316 Sample Paper 1 Timothy Murphy April 19, 2015 Attempt 5 questions. All carry the same mark. 1. State and prove the Fundamental Theorem of Arithmetic (for N). Prove that there are an infinity of primes 3 mod 4. What can you say about primes 1 mod 4? Answer: (a) The integer p > 1 is said to be prime if its only factors are 1 and p itself. Theorem. Each integer n > 1 is expressible as a product of primes, n = p 1... p r, and the expression is unique up to order. Proof. We say that m, n Z are coprime if the only common factor they have is 1. Lemma. If m, n are coprime then we can find x, y Z such that mx + ny = 1. Proof. The result is trivial if m = 0 or n = 0, so we may assume m, n > 0. Consider the set of integers S = {mx + ny : x, y Z}. Let d be the smallest integer > 0 in this set. Divide m by d: m = qd + r, where 0 r < d. Then r S. Hence r = 0 by the minimality of d, ie d m. Similarly d n. Hence d = 1 since m, n are coprime.

2 Lemma. [Euclid s Lemma] Suppose p is prime, and a, b Z. Then p ab = p a or p b. Proof. Suppose p a. Then a, p are coprime, and so there exist x, y Z such that ax + py = 1. Multiplying by b, abx + pby = b = p b, since p divides both terms on the left. Lemma. Every n > 1 is a product of primes. Proof by induction on n. Suppose n is not a prime. Then n = ab, with 1 < a, b < n. Both a and b are expressible as products of primes, by the inductive hypothesis. Hence so is n. Lemma. The expression for n > 1 as a product of primes is unique up to order. Proof by induction on n. Suppose n = p 1 p r = q 1 q s are two expressions for n as products of primes. application of Euclid s Lemma, By repeated p 1 q j for some j. Since q j is prime, it follows that Thus p 1 = q j. n p 1 = p 2 p r = q 1 q j 1 q j+1 q s ; and the result follows from the inductive hypothesis.

3 (b) Suppose the only primes 3 mod 4 are Let Note that By the Fundamental Theorem, p 1,..., p r. N = 4p 1 p r 1. N 3 mod 4. N = q 1 q s where the q s are primes. Then one (at least) of these primes, q j say, must be 3 mod 4. For q 1 q s 1 mod 4 = N 1 mod 4. Thus for some i. But this implies that which is impossible since q j = p i p i N, N 1 mod p i. (c) By Dirichlet s Theorem, there are an infinity of primes 1 mod 4. In fact, if π 1 (n), π 3 (n) are the number of primes p n congruent, respectively, to 1 and 3 mod4 then π 1 (n) π 3 (n) n 2 ln n as n. 2. Given m, n N with gcd(m, n) = 1 and r, s Z, prove that there exists x Z such that x r mod m, x s mod n. Find the smallest positive integer x such that x 3 mod 5, x 7 mod 11, x 12 mod 13. Find the largest integer x not expressible in the form with a, b 0. Answer: x = 7a + 11b

4 (a) Consider the group homomorphism Θ : x mod mn (x mod m, x mod n) : Z/(mn) Z/(m) Z/(n). This homomorphism is injective; for x ker Θ = m x, n x = mn x = x = 0 mod mn. Since Z/(mn) and Z/(m) Z/(n) both contain mn elements, Θ is bijective. In particular, it is surjective; and so we can find x Z/(mn) such that Θ(x) = (r mod m, s mod n). (b) Let us find u, v, w such that u 1 mod 5, u 0 mod 11, u 0 mod 13; v 0 mod 5, v 1 mod 11, v 0 mod 13.w 0 mod 5, w 0 mod 11, w 1 mod 1 For the first, = mod 5, so we can take u = = 286. For the second, 5 13 = 65 1 mod 11, so we can take v = 5 13 = 65. For the third, 5 11 = 55 4 mod 13, so we can take w = = 165.

5 Thus a solution to the 3 simultaneous congruences is x = 3u 4v w, = = The general solution is t = t. Thus the smallest positive solution is x = = 568. (c) Since gcd(7, 11) = 1 we can find x, y Z such that 7x + 11y = 1. In fact so we can take Thus for any n, 7 3 = 21 1 mod 11, x = 3, y = 2. n = 7( 3n) + 11(2n). The general solution to is with t Z. If now then we can choose t so that and then n = 7u + 11v n = 7( 3n + 11t) + 11(2n 7t), n n + 11t < 11, 7( 3n + 11t) < 7 11 = 2n 7t > 0. We have shown therefore that the equation n = 7a + 11b has a solution with a, b 0 if n Obviously there is no such solution if n = 1, so the greatest n with no solution lies between 1 and 76.

6 3. Show that if is prime then a = 2 and e is prime. Find the smallest number (with p prime) that is not prime. Answer: (a) Suppose a > 2. We know that In fact M = a e 1 (a, e > 1) M = 2 p 1 x 1 x e 1. x e 1 = (x 1)(x e 1 + x e 2 + 1) Substituting x = a we see that a 1 a e 1. Now suppose e is not a prime, say where c, d > 1. Then as above, Substituting x = a c, (b) Evidently, e = cd, x 1 x d 1. a c 1 (a c ) d 1 = a e = 3, = 7, = 31, = 127 are all prime. Since 2 10 = 1024, If this is prime then = a mod 2047 for a = 1, 2,..., by Fermat s Little Theorem. In other words, the order of a mod 2047 must divide But the order of 2 mod 2047 is 11, which does not divide Hence M 11 = is not prime.

7 4. Prove that if p is an odd prime, then the multiplicative group (Z/p) is cyclic. Find the orders of all the elements of (Z/17). Answer: (a) Recall that the exponent e of a finite group G is the smallest number e > 1 such that g e = 1 for all g G. In other words, e is the lcm of the orders of the elements of G. By Lagrange s Theorem, e n, the order of G. Lemma. If A is a finite abelian group, and the elements a, b A have coprime orders m, n then the order of ab is mn. Proof. Suppose the order of ab is d. Then d mn since (ab) mn = a mn b mn = 1. On the other hand, (ab) d = 1 = (ab) dn = 1 = a dn b dn = 1 = a dn = 1 = m dn = m d, since m, n are coprime. Similarly n d. Hence since m, n are coprime. Thus mn d, d = mn. Lemma. If the exponent of the finite abelian group A is e then there is an element a A of exponent e.

8 Proof. Suppose e = p e 1 1 p er r. For each i, 1 i n, there must be an element a i whose order is divisible by p e i i. (Otherwise the lcm of the orders would contain p i to a lower power.) Suppose the order of a i is p e i i q i. Then the order of b i = a q i i is p q i i. Hence by the last Lemma, the order of is e. a = b 1 b r Lemma. If F is a finite field of order n then the exponent e of the multiplicative group F satisfies e = n 1. Proof. We have x e = 1 for all x 0 in F. Thus the polynomial f(x) = x e 1 of degree e in F [x] has at least n 1 distinct roots. But a polynomial of degree e has at most e roots. Hence e n 1. On the other hand, by Lagrange s Theorem. Hence e n 1 e = n 1. It follows from the last Lemma that the exponent of (Z/p) is p 1. But then, from the previous Lemma, there is an element in the group of order p 1. Hence the group is cyclic.

9 (b) Recall that if A is a cyclic group of order n, and d n, then: i. There is just one subgroup of order d, it is cyclic, and consists of all elements of order r n; ii. There are φ(d) elements of order d in A. iii. If g generates A then g r generates A if and only if gcd(n, r) = 1. The order of each element of (Z/17) divides 17 1 = 16, in other words the order is 1,2,4,8 or 16. Evidently mod 17 = mod 17. Hence 2 has order 8. Thus the elements of orders 1,2,4 and 8 are the powers of 2, and the remaining elements are of order 16, ie they are primitive roots. So there is 1 element of order 1, namely 1 mod 17; and there is 1 element of order 2, namely 1 = 16 mod 17. There are φ(4) = 2 elements of order 4, namely 2 ±2 = 4, 4 1 mod 17 = ±4 mod 17 = 4, 13 mod 17. There are φ(8) = 4 elements of order 8, namely 2 ±1, 2 ±3 = 2, 8, 8, 2 mod 17 = 2, 8, 9, 15 mod 17. The remaining φ(16) 8 elements, namely are of order 16. [Note that Hence 3, 5, 6, 7, 10, 11, 12, 14 mod mod mod 17. Since 2 1 is of order 8, like 2, it follows that 3 is of order 16.] 5. State and prove Gauss Law of Quadratic Reciprocity. Does there exist an integer x such that x 2 17 mod 30? If there is, find the least such integer 0. Answer:

10 (a) If p is a prime, and a Z is coprime to p, we set ( ) a = p { 1 if there is an x Z such that a x 2 mod p, 1 if there is no such x. Theorem. If p, q are distinct odd primes then ( )( ) { p q 1 if p q 3 mod 4, = q p 1 otherwise. (b) There are many proofs of the Quadratic Reciprocity Theorem. Here is Zolotarev s proof, based on the parity (even or odd) of a permutation. Recall that a permutation π S n is even or odd according as it transforms the alternating polynomial A = i<j(x i x j ) into ±A. We set ɛ(π) = { +1 if π is even 1 if π is odd. Evidently the map π ɛ(π) : (Z/p) {±1} is a homomorphism. We know that every permutation π can be expressed as a product of transpositions. It is easy to see that π is even or odd according as the number of transpositions is even or odd. Also, an even cycle is odd, and an odd cycle is even. Lemma. Suppose p is an odd prime, and a is coprime to p. Let π denote the permutation x ax mod p : (Z/p) (Z/p). Then ( ) a = ɛ(π). p

11 Proof. Recall Eisenstein s Criterion: ( ) a a (p 1)/2 mod p. p ( ) a It follows that = ±1 according as the order of a mod p does p or does not divide (p 1)/2. Suppose the order of a is d. Then the permutation π divides into (p 1)/d cycles of length d. If d (p 1)/2 then (p 1)/d is even, and so ɛ(π) = 1. If d (p 1)/2 then (p 1)/d is odd, and d is even, and so ɛ(π) = 1. Let us arrange the elements 0, 1, 2,..., pq 1. in the form of a p q matrix: 0 1 q 1 q q + 1 2q (p 1)q (p 1)q + 1 pq 1 Thus the matrix contains the element qj + i in position (i, j). For each r [0, pq) let µ(r) denote the remainder of r mod q, ie µ(r) r mod q (0 µ(r) < q). Now let us permute each row in the above matrix, sending qj + i qj + µ(pi). Thus the matrix becomes 0 p q p q q + p 2q p , (p 1)q (p 1)q + p pq p where p = µ(p) Each row has been permuted in the same way, ( and) we have seen p above that the signature of this permutation is. Since there q are an odd number of rows, it follows that the permutation of the matrix elements has signature ( ) p ( ) p p =. q q

12 Notice that each column in the permuted matrix above appears in correct cyclic order, ie if the first element in the ith column is i = µ(pi) then the subsequent elements are q + i, 2q + i,..., (p 1)q +i. Since one of these elements is pi, we can perform a cyclic permutation of the column to bring the elements to pi, q+pi, 2q+ pi,..., (p 1)q + pi (where we are taking all elements modpq). As there are an odd number of elements in each column, each of these cyclic permutations will be even. So the new permutation 0 1 q 1 Π : q q + 1 2q (p 1)q (p 1)q + 1 pq 1 0 p 2p q q + p q + 2p (p 1)q (p 1)q + p (p 1)q + 2p will still have signature ɛ(p i) = ( ) p. q It follows in the same way, on swapping p and q, that the permutation of the q p matrices 0 1 p 1 Π : p p + 1 2p (q 1)p (q 1)p + 1 pq 1 has signature ɛ(p i ) = ( ) q. p Evidently the target matrices in the two cases are transposes of one another. So we have to determine the signature of the permutation Θ : qj + i pi + j defined by the transposition. We know that the signature of a permutation π of {1, 2,..., n} is ( 1) r, where r is the number of inversions, ie the number of u, v with u < v n and π(u) > π(v). In our case (i, j) = qi + j < (i, j ) = qi + j if i < i or i = i and j < j. 0 q 2q p p + q p + 2q (q 1)p (q 1)p + q (q 1)p + 2q

13 We have to determine in these cases if [i, j] = pj + i < [i, j ] = pj + i. Thus we have to determine the number of i, j with i < i and j > j. This number is ((p 1) + (p 2) + + 1)) ((q 1) + (q 2) + + q)) = p(p 1)/2 q(q 1)/2. Since p, q are odd, it follows that ɛ(θ) = ( 1) (p 1)/2 (q 1)/2. Since the result follows: Π = ΠΘ, ɛ(π ) = ɛ(π)ɛ(θ), ie ie ( ) q = p ( ) q p ( ) q ( 1) (p 1)/2 (q 1)/2, p ( ) q = ( 1) (p 1)/2 (q 1)/2. p (c) By the Chinese Remainder Theorem there will exist such an integer if each of the congruences x 2 17 mod 2, y 2 17 mod 3, z 2 17 mod 5, is soluble. The second is not soluble, since 17 2 mod 3, and ( ) 2 = 1. 3 Hence the given congruence is not soluble.

14 6. Prove that the ring Γ of gaussian integers m + ni is a Unique Factorisation Domain, and determine the units and primes in this domain. Show that an integer n > 0 can be expressed in the form n = a 2 + b 2 (a, b N) if and only if each prime p 3 mod 4 divides n to an even power. In how many ways can 1 million be expressed as a sum of two squares? Answer: (a) If z = x + yi, where x, y R, we set z = x yi, and It is readily established that N (z) = z z = x 2 + y 2. i. N (z) Q; ii. N (z) 0 and N (z) = 0 z = 0; iii. If z Γ then N (z) N. iv. N (zw) = N (z)n (w); v. If a Q then N (a) = a 2 ; Lemma. Suppose z, w Γ, with w 0. Then we can find q, r Γ such that z = qw + r, with N (r) < N (w). Proof. Suppose z w = x + iy, where x, y Q. Let m, n Z be the nearest integers to x, y, respectively. Then x m 1 2, y n 1 2. Set Then q = m + in. z q = (x m) + i(y n). w

15 Thus N ( z w 1) = (x m)2 + (y n) = 1 2 < 1. But N ( z w qw 1) = N (z w ) N (z qw) =. N (w) Hence N (z qw) < N (w), from which the result follows on setting r = z qw. Lemma. Any two numbers z, w Γ have a greatest common divisor δ such that δ z, w and δ z, w = δ δ. Also, δ is uniquely defined up to multiplication by a unit. Moreover, there exists u, v Γ such that uz + vw = δ. Proof. We follow the classic Euclidean Algorithm, except that we use N (z) in place of n. We start by dividing z by w: z = q 0 w + r 0, N (r 0 ) < N (w). If r 0 = 0, we are done. Otherwise we divide w by r 0 : w = q 1 r 0 + r 1, N (r 1 ) < N (r 0 ). f r 1 = 0, we are done. Otherwise we continue in this way. Since N (w) > N (r 0 ) > N (r 1 ) >,

16 and the norms are all positive integers, the algorithm must end, say r i = q i r i 1, r i+1 = 0. Setting we see successively that δ = r i, Conversely, if δ z, w then δ r i 1, r i 2,..., r 0, w, z. δ z, w, r 0, r 1,..., r i = δ. The last part of the Lemma follows as in the classic Euclidean Algorithm; we see successively that r 1, r 2,..., r i = δ are each expressible as linear combinations of z, w with coefficients in Γ. Theorem. Γ is a Unique Factorisation Domain. Proof. First we show that any z Γ is a product of irreducibles, by induction on N (z). If z is a unit or irreducible, we are done. If not, suppose z = wt, where neither w nor t is a unit. Then N (z) = N (w)n (t) = N (w), N (t) < N (z). Hence w, t are products of prime elements, and the result follows. To see that the expression is unique, we must establish the analogue of Euclid s Lemma. The proof is identical to the classic case. Lemma. If π Γ is prime element and z, w Γ then π zw = π z or π w. Proof. If π z then gcd(π, z) = 1. Hence there exist u, v such that uπ + vz = 1.

17 Multiplying by w, Multiplying by w, uπw + vzw = w. Since π divides both terms on the left, π w. Now the proof is as before. Again, we argue by induction on N (z). Suppose z = ɛp 1 p r = ɛ p 1... p s. Then for some i. Hence π 1 π i π i π. Now we can divide both sides by π 1 and apply the inductive hypothesis. (b) Lemma. e Γ is a unit if and only if N (e) = 1. Proof. If e is a unit, ie ef = 1 for some f Γ, then N (ef) = 1 = N (e) = N (f) = 1. Conversely, if N (e) = 1 then eē = 1, and so e is a unit, since ē Γ. It follows that e = m + ni is a unit if and only if m 2 + n 2 = 1. Evidently the only solutions to this are (m, n) = (±1, 0), (0, ±1). Thus the only units in Γ are ±1, ±i. (c) Lemma. 1 mod 4. An odd prime p N splits in Γ if and only if p Proof. Suppose p splits, say p = π 1 π r. Then p 2 = N (p) = N (p 1 ) N (pi r ).

18 It follows (from prime factorization in N) that r = 2 and Let π = π 1 = m + ni. Then N (π 1 ) = N (π 2 ) = p. N (π) = m 2 + n 2 = p. Clearly n is coprime to p. So if n 1 denotes the inverse of n modulo p then (mn 1 ) mod p. Hence 1 is a quadratic residue modulo p. But we know (from Euler s Criterion) that this holds if and only if p 1 mod 4. So p remains prime in Γ if p 3 mod 4. Suppose p 1 mod 4. Then there is an r such that ie If p does not split then which is absurd. Finally, r mod p, (r + i)(r i) = pm. p r ± i = p 1, 2 = i(1 i) 2. Thus 2 ramifies in Γ, ie splits into two equal primes. These give all the primes in Γ; for if π is a prime and then π p i for some i. (d) Suppose N (π) = n = p 1 p r n = a 2 + b 2, and suppose p 3 mod 4 divides n. Then it follows from the argument above that p a, b; for otherwise 1 would be a quadratic residue modulo p. Thus p 2 n, and n/p 2 = (a/p) 2 + (b/p) 2.

19 We deduce, on repeating this argument, that p divides n to an even power. Now suppose n = 2 e p e 1 1 p er r q 2f 1 1 q 2fs s, where p i 1 mod 4, q j 3 mod 4. If now p i = π i π i. set Then z = a + ib = (1 i) e π e 1 1 π er r q f 1 1 q fr s. N (z) = a 2 + b 2 = n. (e) Suppose = = a 2 + b 2. We shall assume that a, b 0, and that a b. argument a + ib = f(1 i) 6 (2 + i) s (2 i) t, By the above where f is a unit and r + s = 6. The unit f is uniquely defined by the conditions a, b 0, a b, Hence there are 7 different ways of expressing as a sum of two squares. 7. Define an algebraic number and an algebraic integer. Show that the algebraic numbers form a field, and the algebraic integers form a commutative ring. Prove that ( 2 + 3)/2 is not an algebraic integer. Answer: (a) We say that α C is an algebraic number if it satisfies an equation with a 1,..., a n Q. x n + a 1 x n a n = 0 (b) We say that α is an algebraic integer if it satisfies an equation with a 1,..., a n Z. (c) Lemma. Suppose x n + a 1 x n a n = 0 αv V, where V C is a finite-dimensional vector space. Then α is an algebraic number.

20 Proof. Let e 1,..., e n be a basis for V. Then αe 1 = a 11 e a 1n e n, αe 2 = a 21 e a 2n e n,... αe n = a 11 e a 1n e n, where a ij Q. It follows that α satisfies the polynomial equation det(xi A) = 0. This has rational coefficients. Hence α is algebraic. Now suppose α, β are algebraic, satisfying the equations x m + a 1 x m a m = 0, x n + b 1 x n b n = 0. Consider the vector subspace V C over Q spanned by the mn numbers α i β j (1 i m, 1 j n). It is readily verified that It follows that αv V, βv V. (α + β)v V, (αβ)v V. Hence α + β, αβ are algebraic. Since it is easy to see that α 1 is algebraic, it follows that the algebraic numbers form a field. (d) Lemma. Suppose αa A, where A C is a finitely-generated abelian group Then α is an algebraic integer. Proof. This follows in the same way as the last Lemma, with α satisfying an equation det(xi A) = 0, where now the coefficients are integers.

21 (e) Suppose α = ( 2 + 3)/2 is an algebraic integer. We know that 2 and 3 are algebraic integers. Hence so is 2 3; and so therefore is α( 2 3) = 1 2. Suppose 1/2 satisfies the equation x n + a 1 x n a n = 0 with a 1,..., a n Z. Multiplying by 2 n, 1 + 2a 1 + 4a n a n = 0 = Show that the ring Z[ 3] formed by the numbers m + n 3 (m, n Z) is a Unique Factorisation Domain. Determine the units and primes in this domain. Is Z[ 6] a Unique Factorisation Domain? Answer: (a) Let A = Z[ 3] = {m + n 3 : m, n Z}. The numbers {x + y 3 : x, y Q} form a field Q( 3). (Recall that A is the ring of algebraic integers in this field.) If z = x+y 3 we set z = x y 3, and N (()z) = z z = x 2 3y 2. Lemma. that with Given z, w A with w 0 we can find q, r A such z = qw + r N (()r) < N (()q).

22 Proof. Let z w = x + y 3, with x, y Q. We can find m, n Z such that x m 1 2, y n 1 2. Choose Then q = m + ni. 3 4 N (() z w q) 1 4. It follows from the multiplicative property of the norm that N (()z qw) 3 N (q), 4 and the result follows on setting r = z qw. This Lemma allows us to set up the Euclidean Algorithm in A, and so define gcd(z, w) = δ for z, wina. Moreover, it follows by reversing the algorithm that we can find u, v A such that uz + vw = δ. The analogue of Euclid s Lemma follows: if π Γ is irreducible then π zw = π z or π w. Any z Γ can be expressed as a product of irreducibles. For z = w 1 w 2 w r = N (()z) = N (()w 1 )N (()w 2 ) N (()w r ), so the number of w i in such a product is limited by the number of factors of N (()z). Finally, the uniqueness of the factorisation into irreducibles (up to order) follows in the familiar way from Euclid s Lemma. (b) It is easy to see that z = m + n 3 is a unit in A if and only if For N (()z) = ±1. zw = 1 = N (()z)n (()w) = N (()1) = 1 = N (()z) = N (()w) = ±1.

23 Evidently is a unit, since = 1. It follows that ɛ = ±ɛ n are units, for all n Z. These are in fact the only units. For suppose η is a unit 1. We may assume that η > 1, since just one of ±η, ±η 1 (0, ). Suppose Then Suppose where m, n Z. Then ɛ n η < ɛ n+1. θ = ηɛ n [1, η). θ = m + n 3, m n 3 = ±θ 1. Thus 1 m + n 3 < 2 + 3, 1 m n 3 1. Adding, Thus Since it follows that 0 m < (1 + 3)/2. m = 0 or 1. m 2 3n 2 = ±1 m = 1, n = 0 = θ = 1.

24 (c) Having established unique factorisation in A we may refer to irreducibles as primes. Suppose p Z is a rational prime. Then p factorizes into at most 2 primes in A, since p = π 1 π r = N (()π 1 ) N (()π r ) = N (()p) = p 2, and N (()π i ) > 1 since N (()z) = 1 implies that z is a unit. Conversely, each prime π A is a factor of a unique rational prime p. For if N (()π) = ππ = p 1 p r then π divides one of the p i ; and it cannot divide two different rational primes p, q since we can find x, y Z such that and so px + qy = 1, π p, q = π 1, which is absurd. Also, if a rational prime p splits in Γ then p = ±π π, ie p splits into conjugate primes. For p = ππ = N (()π)n (()π ) = Norm(p) = p 2 = N (()π) = ππ = ±p. Thus we have to determine which rational primes p N split in A. Theorem. i. 3 ramifies (ie splits into two equal primes) in A: ii. 3 = ( 3) 2. Lemma. Suppose p N is a rational prime. Then we can find x Z such that x 2 3 mod p if and only if either p = 2 or 3, or p ±1 mod 12.

25 Proof. The result is trivial if p = 2 or 3. If p 2, 3, then by Gauss Quadratic Reciprocity Law, ( ) ( ) p 3 if p 1 mod 4 3 = ( ) p p if p 3 mod 4 3 and ( ) { p 1 if p 1 mod 3 = 3 1 if p 2 mod 3. Suppose p is a rational prime. If p 3 mod 4 then p cannot split in Γ. For if p splits then p = N (()π) from above; but if π = m+ni then p = N (()π) = m 2 + n 2, and this is impossible if p 3 mod 4 since m 2, n 2 0 or 1 mod 4. On the other hand, if p 1 mod 4 then it does split. For we know in this case that ( ) 1 = 1, p ie we can find n Z such that But p n n = (n + i)(n i) in Γ. Thus if p remained prime in Γ we would have p n + i or p n i, both of which are impossible. Finally, 2 = i(1 + i) 2. Thus 2 ramifies in Γ, ie splits into 2 equal (or associated) primes. (d) Lemma. The integer n N is expressible as a sum of squares if and only if each prime factor p 3 mod 4 occurs to an even power in n Thus 99 =

26 is not expressible as a sum of 2 squares, since 11 3 mod 4 and this occurs only once. Similarly 999 = is not expressible as a sum of 2 squares, since 3 occurs 3 times. Again, 2010 is divisible by 3 but not by 9, and so is not expressible as a sum of 2 squares. Finally, 2317 = is not expressible as a sum of 2 squares, since 7 occurs only once. (Note that it is not necessary to know that 331 is prime; it is sufficient to observe that it is not divisible by 7.)

Proposition The gaussian numbers form a field. The gaussian integers form a commutative ring.

Proposition The gaussian numbers form a field. The gaussian integers form a commutative ring. Chapter 11 Gaussian Integers 11.1 Gaussian Numbers Definition 11.1. A gaussian number is a number of the form z = x + iy (x, y Q). If x, y Z we say that z is a gaussian integer. Proposition 11.1. The gaussian

More information

Part II. Number Theory. Year

Part II. Number Theory. Year Part II Year 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2017 Paper 3, Section I 1G 70 Explain what is meant by an Euler pseudoprime and a strong pseudoprime. Show that 65 is an Euler

More information

Chapter 1. From Euclid to Gauss. 1.1 Prime numbers. If a, b Z we say that a divides b (or is a divisor of b) and we write a b, if.

Chapter 1. From Euclid to Gauss. 1.1 Prime numbers. If a, b Z we say that a divides b (or is a divisor of b) and we write a b, if. Chapter 1 From Euclid to Gauss 1.1 Prime numbers If a, b Z we say that a divides b (or is a divisor of b) and we write a b, if for some c Z. Thus 2 0 but 0 2. b = ac Definition 1.1. The number p N is said

More information

The Chinese Remainder Theorem

The Chinese Remainder Theorem Chapter 5 The Chinese Remainder Theorem 5.1 Coprime moduli Theorem 5.1. Suppose m, n N, and gcd(m, n) = 1. Given any remainders r mod m and s mod n we can find N such that N r mod m and N s mod n. Moreover,

More information

Chapter 5. Modular arithmetic. 5.1 The modular ring

Chapter 5. Modular arithmetic. 5.1 The modular ring Chapter 5 Modular arithmetic 5.1 The modular ring Definition 5.1. Suppose n N and x, y Z. Then we say that x, y are equivalent modulo n, and we write x y mod n if n x y. It is evident that equivalence

More information

Public-key Cryptography: Theory and Practice

Public-key Cryptography: Theory and Practice Public-key Cryptography Theory and Practice Department of Computer Science and Engineering Indian Institute of Technology Kharagpur Chapter 2: Mathematical Concepts Divisibility Congruence Quadratic Residues

More information

Definitions. Notations. Injective, Surjective and Bijective. Divides. Cartesian Product. Relations. Equivalence Relations

Definitions. Notations. Injective, Surjective and Bijective. Divides. Cartesian Product. Relations. Equivalence Relations Page 1 Definitions Tuesday, May 8, 2018 12:23 AM Notations " " means "equals, by definition" the set of all real numbers the set of integers Denote a function from a set to a set by Denote the image of

More information

Mathematics for Cryptography

Mathematics for Cryptography Mathematics for Cryptography Douglas R. Stinson David R. Cheriton School of Computer Science University of Waterloo Waterloo, Ontario, N2L 3G1, Canada March 15, 2016 1 Groups and Modular Arithmetic 1.1

More information

MATH 3030, Abstract Algebra FALL 2012 Toby Kenney Midyear Examination Friday 7th December: 7:00-10:00 PM

MATH 3030, Abstract Algebra FALL 2012 Toby Kenney Midyear Examination Friday 7th December: 7:00-10:00 PM MATH 3030, Abstract Algebra FALL 2012 Toby Kenney Midyear Examination Friday 7th December: 7:00-10:00 PM Basic Questions 1. Compute the factor group Z 3 Z 9 / (1, 6). The subgroup generated by (1, 6) is

More information

The Fundamental Theorem of Arithmetic

The Fundamental Theorem of Arithmetic Chapter 1 The Fundamental Theorem of Arithmetic 1.1 Primes Definition 1.1. We say that p N is prime if it has just two factors in N, 1 and p itself. Number theory might be described as the study of the

More information

φ(xy) = (xy) n = x n y n = φ(x)φ(y)

φ(xy) = (xy) n = x n y n = φ(x)φ(y) Groups 1. (Algebra Comp S03) Let A, B and C be normal subgroups of a group G with A B. If A C = B C and AC = BC then prove that A = B. Let b B. Since b = b1 BC = AC, there are a A and c C such that b =

More information

Course 2BA1: Trinity 2006 Section 9: Introduction to Number Theory and Cryptography

Course 2BA1: Trinity 2006 Section 9: Introduction to Number Theory and Cryptography Course 2BA1: Trinity 2006 Section 9: Introduction to Number Theory and Cryptography David R. Wilkins Copyright c David R. Wilkins 2006 Contents 9 Introduction to Number Theory and Cryptography 1 9.1 Subgroups

More information

Elementary Algebra Chinese Remainder Theorem Euclidean Algorithm

Elementary Algebra Chinese Remainder Theorem Euclidean Algorithm Elementary Algebra Chinese Remainder Theorem Euclidean Algorithm April 11, 2010 1 Algebra We start by discussing algebraic structures and their properties. This is presented in more depth than what we

More information

MATH 152 Problem set 6 solutions

MATH 152 Problem set 6 solutions MATH 52 Problem set 6 solutions. Z[ 2] is a Euclidean domain (i.e. has a division algorithm): the idea is to approximate the quotient by an element in Z[ 2]. More precisely, let a+b 2, c+d 2 Z[ 2] (of

More information

LECTURE 4: CHINESE REMAINDER THEOREM AND MULTIPLICATIVE FUNCTIONS

LECTURE 4: CHINESE REMAINDER THEOREM AND MULTIPLICATIVE FUNCTIONS LECTURE 4: CHINESE REMAINDER THEOREM AND MULTIPLICATIVE FUNCTIONS 1. The Chinese Remainder Theorem We now seek to analyse the solubility of congruences by reinterpreting their solutions modulo a composite

More information

Math 120 HW 9 Solutions

Math 120 HW 9 Solutions Math 120 HW 9 Solutions June 8, 2018 Question 1 Write down a ring homomorphism (no proof required) f from R = Z[ 11] = {a + b 11 a, b Z} to S = Z/35Z. The main difficulty is to find an element x Z/35Z

More information

Math 2070BC Term 2 Weeks 1 13 Lecture Notes

Math 2070BC Term 2 Weeks 1 13 Lecture Notes Math 2070BC 2017 18 Term 2 Weeks 1 13 Lecture Notes Keywords: group operation multiplication associative identity element inverse commutative abelian group Special Linear Group order infinite order cyclic

More information

Algebraic structures I

Algebraic structures I MTH5100 Assignment 1-10 Algebraic structures I For handing in on various dates January March 2011 1 FUNCTIONS. Say which of the following rules successfully define functions, giving reasons. For each one

More information

Chapter 12. Algebraic numbers and algebraic integers Algebraic numbers

Chapter 12. Algebraic numbers and algebraic integers Algebraic numbers Chapter 12 Algebraic numbers and algebraic integers 12.1 Algebraic numbers Definition 12.1. A number α C is said to be algebraic if it satisfies a polynomial equation with rational coefficients a i Q.

More information

Math 312/ AMS 351 (Fall 17) Sample Questions for Final

Math 312/ AMS 351 (Fall 17) Sample Questions for Final Math 312/ AMS 351 (Fall 17) Sample Questions for Final 1. Solve the system of equations 2x 1 mod 3 x 2 mod 7 x 7 mod 8 First note that the inverse of 2 is 2 mod 3. Thus, the first equation becomes (multiply

More information

School of Mathematics

School of Mathematics School of Mathematics Programmes in the School of Mathematics Programmes including Mathematics Final Examination Final Examination 06 22498 MSM3P05 Level H Number Theory 06 16214 MSM4P05 Level M Number

More information

Elementary Number Theory Review. Franz Luef

Elementary Number Theory Review. Franz Luef Elementary Number Theory Review Principle of Induction Principle of Induction Suppose we have a sequence of mathematical statements P(1), P(2),... such that (a) P(1) is true. (b) If P(k) is true, then

More information

MATH 4400 SOLUTIONS TO SOME EXERCISES. 1. Chapter 1

MATH 4400 SOLUTIONS TO SOME EXERCISES. 1. Chapter 1 MATH 4400 SOLUTIONS TO SOME EXERCISES 1.1.3. If a b and b c show that a c. 1. Chapter 1 Solution: a b means that b = na and b c that c = mb. Substituting b = na gives c = (mn)a, that is, a c. 1.2.1. Find

More information

Mathematics Course 111: Algebra I Part I: Algebraic Structures, Sets and Permutations

Mathematics Course 111: Algebra I Part I: Algebraic Structures, Sets and Permutations Mathematics Course 111: Algebra I Part I: Algebraic Structures, Sets and Permutations D. R. Wilkins Academic Year 1996-7 1 Number Systems and Matrix Algebra Integers The whole numbers 0, ±1, ±2, ±3, ±4,...

More information

0 Sets and Induction. Sets

0 Sets and Induction. Sets 0 Sets and Induction Sets A set is an unordered collection of objects, called elements or members of the set. A set is said to contain its elements. We write a A to denote that a is an element of the set

More information

18. Cyclotomic polynomials II

18. Cyclotomic polynomials II 18. Cyclotomic polynomials II 18.1 Cyclotomic polynomials over Z 18.2 Worked examples Now that we have Gauss lemma in hand we can look at cyclotomic polynomials again, not as polynomials with coefficients

More information

Course MA2C02, Hilary Term 2013 Section 9: Introduction to Number Theory and Cryptography

Course MA2C02, Hilary Term 2013 Section 9: Introduction to Number Theory and Cryptography Course MA2C02, Hilary Term 2013 Section 9: Introduction to Number Theory and Cryptography David R. Wilkins Copyright c David R. Wilkins 2000 2013 Contents 9 Introduction to Number Theory 63 9.1 Subgroups

More information

Galois theory (Part II)( ) Example Sheet 1

Galois theory (Part II)( ) Example Sheet 1 Galois theory (Part II)(2015 2016) Example Sheet 1 c.birkar@dpmms.cam.ac.uk (1) Find the minimal polynomial of 2 + 3 over Q. (2) Let K L be a finite field extension such that [L : K] is prime. Show that

More information

Summary Slides for MATH 342 June 25, 2018

Summary Slides for MATH 342 June 25, 2018 Summary Slides for MATH 342 June 25, 2018 Summary slides based on Elementary Number Theory and its applications by Kenneth Rosen and The Theory of Numbers by Ivan Niven, Herbert Zuckerman, and Hugh Montgomery.

More information

Lecture notes: Algorithms for integers, polynomials (Thorsten Theobald)

Lecture notes: Algorithms for integers, polynomials (Thorsten Theobald) Lecture notes: Algorithms for integers, polynomials (Thorsten Theobald) 1 Euclid s Algorithm Euclid s Algorithm for computing the greatest common divisor belongs to the oldest known computing procedures

More information

Polynomials. Chapter 4

Polynomials. Chapter 4 Chapter 4 Polynomials In this Chapter we shall see that everything we did with integers in the last Chapter we can also do with polynomials. Fix a field F (e.g. F = Q, R, C or Z/(p) for a prime p). Notation

More information

A Guide to Arithmetic

A Guide to Arithmetic A Guide to Arithmetic Robin Chapman August 5, 1994 These notes give a very brief resumé of my number theory course. Proofs and examples are omitted. Any suggestions for improvements will be gratefully

More information

ECEN 5022 Cryptography

ECEN 5022 Cryptography Elementary Algebra and Number Theory University of Colorado Spring 2008 Divisibility, Primes Definition. N denotes the set {1, 2, 3,...} of natural numbers and Z denotes the set of integers {..., 2, 1,

More information

PRACTICE FINAL MATH , MIT, SPRING 13. You have three hours. This test is closed book, closed notes, no calculators.

PRACTICE FINAL MATH , MIT, SPRING 13. You have three hours. This test is closed book, closed notes, no calculators. PRACTICE FINAL MATH 18.703, MIT, SPRING 13 You have three hours. This test is closed book, closed notes, no calculators. There are 11 problems, and the total number of points is 180. Show all your work.

More information

Number Theory Solutions Packet

Number Theory Solutions Packet Number Theory Solutions Pacet 1 There exist two distinct positive integers, both of which are divisors of 10 10, with sum equal to 157 What are they? Solution Suppose 157 = x + y for x and y divisors of

More information

Homework #2 solutions Due: June 15, 2012

Homework #2 solutions Due: June 15, 2012 All of the following exercises are based on the material in the handout on integers found on the class website. 1. Find d = gcd(475, 385) and express it as a linear combination of 475 and 385. That is

More information

Theorems and Definitions in Group Theory

Theorems and Definitions in Group Theory Theorems and Definitions in Group Theory Shunan Zhao Contents 1 Basics of a group 3 1.1 Basic Properties of Groups.......................... 3 1.2 Properties of Inverses............................. 3

More information

The primitive root theorem

The primitive root theorem The primitive root theorem Mar Steinberger First recall that if R is a ring, then a R is a unit if there exists b R with ab = ba = 1. The collection of all units in R is denoted R and forms a group under

More information

PRIME NUMBERS YANKI LEKILI

PRIME NUMBERS YANKI LEKILI PRIME NUMBERS YANKI LEKILI We denote by N the set of natural numbers: 1,2,..., These are constructed using Peano axioms. We will not get into the philosophical questions related to this and simply assume

More information

Congruences and Residue Class Rings

Congruences and Residue Class Rings Congruences and Residue Class Rings (Chapter 2 of J. A. Buchmann, Introduction to Cryptography, 2nd Ed., 2004) Shoichi Hirose Faculty of Engineering, University of Fukui S. Hirose (U. Fukui) Congruences

More information

ALGEBRA I (LECTURE NOTES 2017/2018) LECTURE 9 - CYCLIC GROUPS AND EULER S FUNCTION

ALGEBRA I (LECTURE NOTES 2017/2018) LECTURE 9 - CYCLIC GROUPS AND EULER S FUNCTION ALGEBRA I (LECTURE NOTES 2017/2018) LECTURE 9 - CYCLIC GROUPS AND EULER S FUNCTION PAVEL RŮŽIČKA 9.1. Congruence modulo n. Let us have a closer look at a particular example of a congruence relation on

More information

1. Factorization Divisibility in Z.

1. Factorization Divisibility in Z. 8 J. E. CREMONA 1.1. Divisibility in Z. 1. Factorization Definition 1.1.1. Let a, b Z. Then we say that a divides b and write a b if b = ac for some c Z: a b c Z : b = ac. Alternatively, we may say that

More information

CHAPTER 6. Prime Numbers. Definition and Fundamental Results

CHAPTER 6. Prime Numbers. Definition and Fundamental Results CHAPTER 6 Prime Numbers Part VI of PJE. Definition and Fundamental Results 6.1. Definition. (PJE definition 23.1.1) An integer p is prime if p > 1 and the only positive divisors of p are 1 and p. If n

More information

Exercises MAT2200 spring 2014 Ark 5 Rings and fields and factorization of polynomials

Exercises MAT2200 spring 2014 Ark 5 Rings and fields and factorization of polynomials Exercises MAT2200 spring 2014 Ark 5 Rings and fields and factorization of polynomials This Ark concerns the weeks No. (Mar ) andno. (Mar ). Status for this week: On Monday Mar : Finished section 23(Factorization

More information

1 Overview and revision

1 Overview and revision MTH6128 Number Theory Notes 1 Spring 2018 1 Overview and revision In this section we will meet some of the concerns of Number Theory, and have a brief revision of some of the relevant material from Introduction

More information

A. Algebra and Number Theory

A. Algebra and Number Theory A. Algebra and Number Theory Public-key cryptosystems are based on modular arithmetic. In this section, we summarize the concepts and results from algebra and number theory which are necessary for an understanding

More information

Modern Algebra I. Circle the correct answer; no explanation is required. Each problem in this section counts 5 points.

Modern Algebra I. Circle the correct answer; no explanation is required. Each problem in this section counts 5 points. 1 2 3 style total Math 415 Please print your name: Answer Key 1 True/false Circle the correct answer; no explanation is required. Each problem in this section counts 5 points. 1. Every group of order 6

More information

4 PRIMITIVE ROOTS Order and Primitive Roots The Index Existence of primitive roots for prime modulus...

4 PRIMITIVE ROOTS Order and Primitive Roots The Index Existence of primitive roots for prime modulus... PREFACE These notes have been prepared by Dr Mike Canfell (with minor changes and extensions by Dr Gerd Schmalz) for use by the external students in the unit PMTH 338 Number Theory. This booklet covers

More information

Congruent Number Problem and Elliptic curves

Congruent Number Problem and Elliptic curves Congruent Number Problem and Elliptic curves December 12, 2010 Contents 1 Congruent Number problem 2 1.1 1 is not a congruent number.................................. 2 2 Certain Elliptic Curves 4 3 Using

More information

Elementary Number Theory MARUCO. Summer, 2018

Elementary Number Theory MARUCO. Summer, 2018 Elementary Number Theory MARUCO Summer, 2018 Problem Set #0 axiom, theorem, proof, Z, N. Axioms Make a list of axioms for the integers. Does your list adequately describe them? Can you make this list as

More information

Chapter 4. Characters and Gauss sums. 4.1 Characters on finite abelian groups

Chapter 4. Characters and Gauss sums. 4.1 Characters on finite abelian groups Chapter 4 Characters and Gauss sums 4.1 Characters on finite abelian groups In what follows, abelian groups are multiplicatively written, and the unit element of an abelian group A is denoted by 1 or 1

More information

Quasi-reducible Polynomials

Quasi-reducible Polynomials Quasi-reducible Polynomials Jacques Willekens 06-Dec-2008 Abstract In this article, we investigate polynomials that are irreducible over Q, but are reducible modulo any prime number. 1 Introduction Let

More information

Math 109 HW 9 Solutions

Math 109 HW 9 Solutions Math 109 HW 9 Solutions Problems IV 18. Solve the linear diophantine equation 6m + 10n + 15p = 1 Solution: Let y = 10n + 15p. Since (10, 15) is 5, we must have that y = 5x for some integer x, and (as we

More information

A field F is a set of numbers that includes the two numbers 0 and 1 and satisfies the properties:

A field F is a set of numbers that includes the two numbers 0 and 1 and satisfies the properties: Byte multiplication 1 Field arithmetic A field F is a set of numbers that includes the two numbers 0 and 1 and satisfies the properties: F is an abelian group under addition, meaning - F is closed under

More information

Chapter 4 Finite Fields

Chapter 4 Finite Fields Chapter 4 Finite Fields Introduction will now introduce finite fields of increasing importance in cryptography AES, Elliptic Curve, IDEA, Public Key concern operations on numbers what constitutes a number

More information

Discrete Math, Second Problem Set (June 24)

Discrete Math, Second Problem Set (June 24) Discrete Math, Second Problem Set (June 24) REU 2003 Instructor: Laszlo Babai Scribe: D Jeremy Copeland 1 Number Theory Remark 11 For an arithmetic progression, a 0, a 1 = a 0 +d, a 2 = a 0 +2d, to have

More information

Definitions, Theorems and Exercises. Abstract Algebra Math 332. Ethan D. Bloch

Definitions, Theorems and Exercises. Abstract Algebra Math 332. Ethan D. Bloch Definitions, Theorems and Exercises Abstract Algebra Math 332 Ethan D. Bloch December 26, 2013 ii Contents 1 Binary Operations 3 1.1 Binary Operations............................... 4 1.2 Isomorphic Binary

More information

(January 14, 2009) q n 1 q d 1. D = q n = q + d

(January 14, 2009) q n 1 q d 1. D = q n = q + d (January 14, 2009) [10.1] Prove that a finite division ring D (a not-necessarily commutative ring with 1 in which any non-zero element has a multiplicative inverse) is commutative. (This is due to Wedderburn.)

More information

NUMBER SYSTEMS. Number theory is the study of the integers. We denote the set of integers by Z:

NUMBER SYSTEMS. Number theory is the study of the integers. We denote the set of integers by Z: NUMBER SYSTEMS Number theory is the study of the integers. We denote the set of integers by Z: Z = {..., 3, 2, 1, 0, 1, 2, 3,... }. The integers have two operations defined on them, addition and multiplication,

More information

MATH 361: NUMBER THEORY FOURTH LECTURE

MATH 361: NUMBER THEORY FOURTH LECTURE MATH 361: NUMBER THEORY FOURTH LECTURE 1. Introduction Everybody knows that three hours after 10:00, the time is 1:00. That is, everybody is familiar with modular arithmetic, the usual arithmetic of the

More information

Part IA. Numbers and Sets. Year

Part IA. Numbers and Sets. Year Part IA Year 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2004 2003 2002 2001 2017 19 Paper 4, Section I 1D (a) Show that for all positive integers z and n, either z 2n 0 (mod 3) or

More information

Algebra. Modular arithmetic can be handled mathematically by introducing a congruence relation on the integers described in the above example.

Algebra. Modular arithmetic can be handled mathematically by introducing a congruence relation on the integers described in the above example. Coding Theory Massoud Malek Algebra Congruence Relation The definition of a congruence depends on the type of algebraic structure under consideration Particular definitions of congruence can be made for

More information

4 Powers of an Element; Cyclic Groups

4 Powers of an Element; Cyclic Groups 4 Powers of an Element; Cyclic Groups Notation When considering an abstract group (G, ), we will often simplify notation as follows x y will be expressed as xy (x y) z will be expressed as xyz x (y z)

More information

x 3 2x = (x 2) (x 2 2x + 1) + (x 2) x 2 2x + 1 = (x 4) (x + 2) + 9 (x + 2) = ( 1 9 x ) (9) + 0

x 3 2x = (x 2) (x 2 2x + 1) + (x 2) x 2 2x + 1 = (x 4) (x + 2) + 9 (x + 2) = ( 1 9 x ) (9) + 0 1. (a) i. State and prove Wilson's Theorem. ii. Show that, if p is a prime number congruent to 1 modulo 4, then there exists a solution to the congruence x 2 1 mod p. (b) i. Let p(x), q(x) be polynomials

More information

2.3 In modular arithmetic, all arithmetic operations are performed modulo some integer.

2.3 In modular arithmetic, all arithmetic operations are performed modulo some integer. CHAPTER 2 INTRODUCTION TO NUMBER THEORY ANSWERS TO QUESTIONS 2.1 A nonzero b is a divisor of a if a = mb for some m, where a, b, and m are integers. That is, b is a divisor of a if there is no remainder

More information

May 6, Be sure to write your name on your bluebook. Use a separate page (or pages) for each problem. Show all of your work.

May 6, Be sure to write your name on your bluebook. Use a separate page (or pages) for each problem. Show all of your work. Math 236H May 6, 2008 Be sure to write your name on your bluebook. Use a separate page (or pages) for each problem. Show all of your work. 1. (15 points) Prove that the symmetric group S 4 is generated

More information

Prime Numbers and Irrational Numbers

Prime Numbers and Irrational Numbers Chapter 4 Prime Numbers and Irrational Numbers Abstract The question of the existence of prime numbers in intervals is treated using the approximation of cardinal of the primes π(x) given by Lagrange.

More information

arxiv:math/ v1 [math.nt] 21 Sep 2004

arxiv:math/ v1 [math.nt] 21 Sep 2004 arxiv:math/0409377v1 [math.nt] 21 Sep 2004 ON THE GCD OF AN INFINITE NUMBER OF INTEGERS T. N. VENKATARAMANA Introduction In this paper, we consider the greatest common divisor (to be abbreviated gcd in

More information

Abstract Algebra, Second Edition, by John A. Beachy and William D. Blair. Corrections and clarifications

Abstract Algebra, Second Edition, by John A. Beachy and William D. Blair. Corrections and clarifications 1 Abstract Algebra, Second Edition, by John A. Beachy and William D. Blair Corrections and clarifications Note: Some corrections were made after the first printing of the text. page 9, line 8 For of the

More information

Introduction to Number Theory 1. c Eli Biham - December 13, Introduction to Number Theory 1

Introduction to Number Theory 1. c Eli Biham - December 13, Introduction to Number Theory 1 Introduction to Number Theory 1 c Eli Biham - December 13, 2012 206 Introduction to Number Theory 1 Division Definition: Let a and b be integers. We say that a divides b, or a b if d s.t. b = ad. If b

More information

TRINITY COLLEGE SCHOOL OF MATHEMATICS

TRINITY COLLEGE SCHOOL OF MATHEMATICS UNIVERSITY OF DUBLIN TRINITY COLLEGE SCHOOL OF MATHEMATICS Evariste Galois 1811-1832 Finite Fields Course MA346D Part I Timothy Murphy Contents 1 The Prime Fields 1 1 2 The Prime Subfield of a Finite Field

More information

Homework 10 M 373K by Mark Lindberg (mal4549)

Homework 10 M 373K by Mark Lindberg (mal4549) Homework 10 M 373K by Mark Lindberg (mal4549) 1. Artin, Chapter 11, Exercise 1.1. Prove that 7 + 3 2 and 3 + 5 are algebraic numbers. To do this, we must provide a polynomial with integer coefficients

More information

LECTURE NOTES IN CRYPTOGRAPHY

LECTURE NOTES IN CRYPTOGRAPHY 1 LECTURE NOTES IN CRYPTOGRAPHY Thomas Johansson 2005/2006 c Thomas Johansson 2006 2 Chapter 1 Abstract algebra and Number theory Before we start the treatment of cryptography we need to review some basic

More information

PUTNAM TRAINING NUMBER THEORY. Exercises 1. Show that the sum of two consecutive primes is never twice a prime.

PUTNAM TRAINING NUMBER THEORY. Exercises 1. Show that the sum of two consecutive primes is never twice a prime. PUTNAM TRAINING NUMBER THEORY (Last updated: December 11, 2017) Remark. This is a list of exercises on Number Theory. Miguel A. Lerma Exercises 1. Show that the sum of two consecutive primes is never twice

More information

Honors Algebra 4, MATH 371 Winter 2010 Assignment 3 Due Friday, February 5 at 08:35

Honors Algebra 4, MATH 371 Winter 2010 Assignment 3 Due Friday, February 5 at 08:35 Honors Algebra 4, MATH 371 Winter 2010 Assignment 3 Due Friday, February 5 at 08:35 1. Let R 0 be a commutative ring with 1 and let S R be the subset of nonzero elements which are not zero divisors. (a)

More information

Some algebraic number theory and the reciprocity map

Some algebraic number theory and the reciprocity map Some algebraic number theory and the reciprocity map Ervin Thiagalingam September 28, 2015 Motivation In Weinstein s paper, the main problem is to find a rule (reciprocity law) for when an irreducible

More information

Algebra Review. Instructor: Laszlo Babai Notes by Vincent Lucarelli and the instructor. June 15, 2001

Algebra Review. Instructor: Laszlo Babai Notes by Vincent Lucarelli and the instructor. June 15, 2001 Algebra Review Instructor: Laszlo Babai Notes by Vincent Lucarelli and the instructor June 15, 2001 1 Groups Definition 1.1 A semigroup (G, ) is a set G with a binary operation such that: Axiom 1 ( a,

More information

Algebraic number theory Solutions to exercise sheet for chapter 4

Algebraic number theory Solutions to exercise sheet for chapter 4 Algebraic number theory Solutions to exercise sheet for chapter 4 Nicolas Mascot n.a.v.mascot@warwick.ac.uk), Aurel Page a.r.page@warwick.ac.uk) TAs: Chris Birkbeck c.d.birkbeck@warwick.ac.uk), George

More information

= 1 2x. x 2 a ) 0 (mod p n ), (x 2 + 2a + a2. x a ) 2

= 1 2x. x 2 a ) 0 (mod p n ), (x 2 + 2a + a2. x a ) 2 8. p-adic numbers 8.1. Motivation: Solving x 2 a (mod p n ). Take an odd prime p, and ( an) integer a coprime to p. Then, as we know, x 2 a (mod p) has a solution x Z iff = 1. In this case we can suppose

More information

Definition List Modern Algebra, Fall 2011 Anders O.F. Hendrickson

Definition List Modern Algebra, Fall 2011 Anders O.F. Hendrickson Definition List Modern Algebra, Fall 2011 Anders O.F. Hendrickson On almost every Friday of the semester, we will have a brief quiz to make sure you have memorized the definitions encountered in our studies.

More information

List of topics for the preliminary exam in algebra

List of topics for the preliminary exam in algebra List of topics for the preliminary exam in algebra 1 Basic concepts 1. Binary relations. Reflexive, symmetric/antisymmetryc, and transitive relations. Order and equivalence relations. Equivalence classes.

More information

Chapter 3. Rings. The basic commutative rings in mathematics are the integers Z, the. Examples

Chapter 3. Rings. The basic commutative rings in mathematics are the integers Z, the. Examples Chapter 3 Rings Rings are additive abelian groups with a second operation called multiplication. The connection between the two operations is provided by the distributive law. Assuming the results of Chapter

More information

Quizzes for Math 401

Quizzes for Math 401 Quizzes for Math 401 QUIZ 1. a) Let a,b be integers such that λa+µb = 1 for some inetegrs λ,µ. Prove that gcd(a,b) = 1. b) Use Euclid s algorithm to compute gcd(803, 154) and find integers λ,µ such that

More information

GRE Subject test preparation Spring 2016 Topic: Abstract Algebra, Linear Algebra, Number Theory.

GRE Subject test preparation Spring 2016 Topic: Abstract Algebra, Linear Algebra, Number Theory. GRE Subject test preparation Spring 2016 Topic: Abstract Algebra, Linear Algebra, Number Theory. Linear Algebra Standard matrix manipulation to compute the kernel, intersection of subspaces, column spaces,

More information

Algebra Qualifying Exam Solutions. Thomas Goller

Algebra Qualifying Exam Solutions. Thomas Goller Algebra Qualifying Exam Solutions Thomas Goller September 4, 2 Contents Spring 2 2 2 Fall 2 8 3 Spring 2 3 4 Fall 29 7 5 Spring 29 2 6 Fall 28 25 Chapter Spring 2. The claim as stated is false. The identity

More information

A Generalization of Wilson s Theorem

A Generalization of Wilson s Theorem A Generalization of Wilson s Theorem R. Andrew Ohana June 3, 2009 Contents 1 Introduction 2 2 Background Algebra 2 2.1 Groups................................. 2 2.2 Rings.................................

More information

D-MATH Algebra II FS18 Prof. Marc Burger. Solution 26. Cyclotomic extensions.

D-MATH Algebra II FS18 Prof. Marc Burger. Solution 26. Cyclotomic extensions. D-MAH Algebra II FS18 Prof. Marc Burger Solution 26 Cyclotomic extensions. In the following, ϕ : Z 1 Z 0 is the Euler function ϕ(n = card ((Z/nZ. For each integer n 1, we consider the n-th cyclotomic polynomial

More information

Math 120: Homework 6 Solutions

Math 120: Homework 6 Solutions Math 120: Homewor 6 Solutions November 18, 2018 Problem 4.4 # 2. Prove that if G is an abelian group of order pq, where p and q are distinct primes then G is cyclic. Solution. By Cauchy s theorem, G has

More information

MINIMAL GENERATING SETS OF GROUPS, RINGS, AND FIELDS

MINIMAL GENERATING SETS OF GROUPS, RINGS, AND FIELDS MINIMAL GENERATING SETS OF GROUPS, RINGS, AND FIELDS LORENZ HALBEISEN, MARTIN HAMILTON, AND PAVEL RŮŽIČKA Abstract. A subset X of a group (or a ring, or a field) is called generating, if the smallest subgroup

More information

Chuck Garner, Ph.D. May 25, 2009 / Georgia ARML Practice

Chuck Garner, Ph.D. May 25, 2009 / Georgia ARML Practice Some Chuck, Ph.D. Department of Mathematics Rockdale Magnet School for Science Technology May 25, 2009 / Georgia ARML Practice Outline 1 2 3 4 Outline 1 2 3 4 Warm-Up Problem Problem Find all positive

More information

2 (17) Find non-trivial left and right ideals of the ring of 22 matrices over R. Show that there are no nontrivial two sided ideals. (18) State and pr

2 (17) Find non-trivial left and right ideals of the ring of 22 matrices over R. Show that there are no nontrivial two sided ideals. (18) State and pr MATHEMATICS Introduction to Modern Algebra II Review. (1) Give an example of a non-commutative ring; a ring without unit; a division ring which is not a eld and a ring which is not a domain. (2) Show that

More information

Chapter 8. P-adic numbers. 8.1 Absolute values

Chapter 8. P-adic numbers. 8.1 Absolute values Chapter 8 P-adic numbers Literature: N. Koblitz, p-adic Numbers, p-adic Analysis, and Zeta-Functions, 2nd edition, Graduate Texts in Mathematics 58, Springer Verlag 1984, corrected 2nd printing 1996, Chap.

More information

D-MATH Algebra I HS 2013 Prof. Brent Doran. Solution 3. Modular arithmetic, quotients, product groups

D-MATH Algebra I HS 2013 Prof. Brent Doran. Solution 3. Modular arithmetic, quotients, product groups D-MATH Algebra I HS 2013 Prof. Brent Doran Solution 3 Modular arithmetic, quotients, product groups 1. Show that the functions f = 1/x, g = (x 1)/x generate a group of functions, the law of composition

More information

Basic elements of number theory

Basic elements of number theory Cryptography Basic elements of number theory Marius Zimand 1 Divisibility, prime numbers By default all the variables, such as a, b, k, etc., denote integer numbers. Divisibility a 0 divides b if b = a

More information

Basic elements of number theory

Basic elements of number theory Cryptography Basic elements of number theory Marius Zimand By default all the variables, such as a, b, k, etc., denote integer numbers. Divisibility a 0 divides b if b = a k for some integer k. Notation

More information

Explicit Methods in Algebraic Number Theory

Explicit Methods in Algebraic Number Theory Explicit Methods in Algebraic Number Theory Amalia Pizarro Madariaga Instituto de Matemáticas Universidad de Valparaíso, Chile amaliapizarro@uvcl 1 Lecture 1 11 Number fields and ring of integers Algebraic

More information

Rings and modular arithmetic

Rings and modular arithmetic Chapter 8 Rings and modular arithmetic So far, we have been working with just one operation at a time. But standard number systems, such as Z, have two operations + and which interact. It is useful to

More information

32 Divisibility Theory in Integral Domains

32 Divisibility Theory in Integral Domains 3 Divisibility Theory in Integral Domains As we have already mentioned, the ring of integers is the prototype of integral domains. There is a divisibility relation on * : an integer b is said to be divisible

More information

Background Material in Algebra and Number Theory. Groups

Background Material in Algebra and Number Theory. Groups PRELIMINARY READING FOR ALGEBRAIC NUMBER THEORY. HT 2016/17. Section 0. Background Material in Algebra and Number Theory The following gives a summary of the main ideas you need to know as prerequisites

More information

ax b mod m. has a solution if and only if d b. In this case, there is one solution, call it x 0, to the equation and there are d solutions x m d

ax b mod m. has a solution if and only if d b. In this case, there is one solution, call it x 0, to the equation and there are d solutions x m d 10. Linear congruences In general we are going to be interested in the problem of solving polynomial equations modulo an integer m. Following Gauss, we can work in the ring Z m and find all solutions to

More information