Examples and Exercises

Size: px
Start display at page:

Download "Examples and Exercises"

Transcription

1 Examples and Exercises Guerino Mazzola January 6, 00 Example of A Rigorous Proof Claim: Let a, b, c be sets. Then we have c (a b) = (c a) (c b). Proof. By definition of equality of sets, we have to prove both inclusions, and.. means: x c (a b) IMPLIES x (c a) (c b). Let us give the proof stepwise:. IF x c (a b) IMPLIES x c AND x a b (by definition of the difference of sets).. x a b IMPLIES x a AND x b (by definition of the union a b) 3. Insert implication. into the implication.: x c (a b) IMPLIES (x c AND x a AND x b) (such logical operations are allowed without altering the truth value). 4. But x c (a b) IMPLIES (x c AND x a AND x b) has the same truth value as x c (a b) IMPLIES ((x c AND x a) AND (x c AND x b)) 5. The latter means, by definition of set difference and intersection that x c (a b) IMPLIES x (c a) (c b). 6. The converse inclusion can also be shown with this rigor, and we have our claim,.

2 Allen Forte s set complexes Let T P, where P is the pitch class set P = {C, C, D, D, E, F, F, G, G, A, A, B}. Forte defines a subset K(T ) P, which he calls the set complex of T, by the attribute S K(T ) iff. S T OR. S T OR In Forte s notation, the symbol X Y stands for X Y OR Y X. Prove that this is equivalent to the following conditions in terms of Boolean algebra operations. S T = S OR. S T = T OR 3. S + T = (S T ) OR 4. S T = Hint for the third condition: S T implies S T = P and therefore S + T = (S T ). On the other hand, if S T is false, then there is an element not in S and not in T, so S T P, therefore S + T (S T ). Therefore S T is equivalent to S + T = (S T ). 3 Relations Take the set a = {r, s, t, u, v} with the mutually different elements r, s, t, u, v. Consider these relations on a:. R = {(r, r), (u, u), (t, t), (v, v), (s, s), (r, s)}. R = {(s, t), (r, s), (t, u), (u, v)} 3. R 3 = a a 4. R 4 = {(r, s), (s, t), (t, u), (u, v), (r, t), (r, u), (r, v), (s, t), (s, u), (s, v), (t, u), (t, v)} 5. R 5 = {(r, s), (t, u)} a {(r, s), (t, u)} Which of these relations is reflexive, transitive, symmetric, linear, an equivalence relation? Take the partition a = {r, v} {s, t} {u} of the above set. Exhibit the equivalence relation on a giving rise to this partition. For any two relations R X, S Y, one defines the Cartesian product relation R S (X Y ) by the condition that ((x, y), (x, y )) R S iff (x, x ) R AND

3 (y, y ) S. Example: Take this Cartesian product ordering on the Cartesian product N N of the natural number set N = {0,,, 3,...} with itself, and with the natural ordering among natural numbers. Prove that this is a partial ordering, but not a linear ordering. Give an example of the violation of the latter condition. Take alternatively the lexicographic ordering on N N (view it as the set N, and = {0, } being ordered naturally by 0 < ). We know that the lexicographic ordering is linear. So exhibit the order relation for that same example. 4 Natural Numbers and Recursion We want to make some examples of the proof by induction technique enabled by the fifth Peano axiom. (We know from the last lecture that addition is associative and shall use this fact now.) Show that for all natural numbers a, b, a + b = b + a. To do so, first, show that a + = + a by induction on a. For a = 0, we have 0 + = = + 0, and if a + = + a holds, then for the successor of a, we have a + + = (a + ) + = ( + a) + = + (a + ) = + a +, and we are done. We then show that a + 0 = 0 + a = a for all a by induction on a. This is evidently true for a = 0, check! And if it holds for a it also holds for its successor. In fact, a = a + = a + = (0 + a) + = 0 + (a + ) = 0 + a +. To prove the statement a + b = b + a, we make induction on a. For a = 0, we have a + b = 0 + b = b + 0 from the above. If a + b = b + a holds, then for the successor of a, we have a + + b = (a + ) + b = a + ( + b) = a + (b + ) = (a + b) + = (b + a) + = b + (a + ), and we are done. Next, we give a proof by induction of the famous formula n n(n + ) i = i=0 for the sum of all natural numbers up to n. This formula was found by yound Carl Friedrich Gauss (the inventor of the complex numbers) while he as a pupil and always annoyed the teacher by solving math problems in no time. So the teacher would ask Gauss to calculate the sum to keep him quiet for a while. But Gauss immediately found the solution by adding + 00, + 99, , etc., So it is 50 0 = We prove the formula by induction on n. It is evidently true for n = 0. Then, suppose it is true for n. We want to prove it for n + = n +. In fact, n+ ( n ) i = i + (n + ) = i=0 i=0 n(n + ) + (n + ) = (n + )(n + ) = (n + )((n + ) + ). (Here we are supposing that the well-known laws of rational number arithmetic have been proved.) 3

4 Next, we want to prove the formula for counting the bijections f : a a of a finite set a onto itself. Such bijecions are also called permutations of the set a. Let us denote the set of bijections by Sym(a), so this is a subset of Set(a, a). The formula to be proved is card(sym(a)) = card(a)! For example, if card(a) = 4, then card(sym(a)) = 4! = 3 4 = 4. The proof of this formula goes by induction on card(a). For the starting value card(a) = 0, i.e., a =, we have Sym(a) = {Id a }, so in fact card(sym( )) = = 0! is the correct formula. To prove the induction step from card(a) = n to card(a) = n +, we do the following. We first fix a bijection u : a n + such that every element x a correponds one-to-one to an element q(x) n +. This means that we index the a-elements by the n + natural numbers from 0 to n. Evidently, we may now as well calculate the permutations of the set n + instead of a. The idea of proof is this one: Each such permutation f : n + n + sends the maximal element n to a number f(n). If we have f(n) = n, f leaves n fixed, which means that f is essentially a permutation of the set n of the first n elements of n +. So there are n! such permutations, by the induction hypothesis. Now, if f(n) = k < n, we may append to f another very simple permutation of n +, namely the exchange of k and n. This one is denoted by (k, n) and is called the transposition of k and n. But then, the composed permutation (k, n) f leaves n fixed, and therefore is one of the already counted n! permutations. Hence we get n! new permutations for all permutations senting n to that k. Now, this k may be any of the n elements of n. We therefore get n such cases, and, counting also the very first case, where n was left fixed, this adds up to n + cases, each of which having n! permutations, all in all n! (n + ) = (n + )!, and we are done. We now want to give a roof by induction of the formula card( a ) = card(a) for the cardinality of the powerset of a finite set a. We proceed by induction on the cardinality of a. The formula evidently holds for card(a) = 0 card(a) =. As before, for the general induction step n to n +, we might just fix a bijection of a with the number n + = card(a) and transfer our discussion to n +. To count the subsets of n +, distinguish those subsets which are already contained in the subset n n +. Their number is, by induction hypothesis, n. The other subsets all contain the element n and are arbitrary besides that condition. So such a subset can be written as x = (x n) {n}. Therefore it is characterized by its intersection x n, so again there are n such subsets. All in all we now have n + n = n = n+ subsets as required. Let us do some examples of the division theorem a = q b+r. For the following numbers a, b, all written in decimal representation, do exhibit the numbers q, r, with 0 r < b:. a = 3, b = 3 4

5 . a = 45, b = 3. a = 55, b = 6 5 Classical Number Domains Consider the 5-adic (!!!) representation of a real number x = , where 43 means that these two entries are repeated until infinity to the right, i.e., x = We know that this must be a rational number u v. Calculate this fraction! Use our method as discussed in class: multiply x by a power 5 m of the basis 5 and subtract x from this power product 5 m x in order to eliminate the periodic repetition And if you do not recall the discussion in class, here is the solution: You first have to multiply x by a power 5 m such that the resulting product 5 m x has the period at the same place as the original number x. Obviously, we may take m = since the period has length, so we get 5 x = Then we subtract x from 5 x: 5 x = x = (5 )x = = So, since 5 = 44, we have(always in 5-adic notation!) x = Prove that the real number 0.9 in the decimal representation equals.0. Proceed as follows: Use first that 0.9 is represented by the Cauchy sequence x 0 = 0, x = 0.90, x = 0.990, x 3 = ,... x n = (the nth number having 9 until the nth position to the right of the dot and 0 after that). Show that the difference sequence.0 x 0,.0 x,.0 x,.0 x 3,....0 x n,... is a zero sequence. This implies that 0.9 =.0. Consider the chromatic octave set χ c = {c, d, d,...b} from c in just tuning (built upon the primes,3,5), as represented by points on the Euler space Q 3,i.e., c = (0, 0, 0), g = (,, 0), etc., see the graphic which was distributed in class. Consider the corresponding octave set χ g built by the same interval distances from g χ c. What is the intersection χ c χ g? Here is the solution, which you may draw from the image which I distributed in class. The intersection has three elements, shown in circles: 5

6 Use the representation of complex numbers x = Re(x)+i Im(x) to prove Re(x) = x+x and Im(x) = x x i. Prove that for complex numbers x, y, we have x y = x y by use of the definition x = x x, and by use of the fact that for any two non-negative real numbers u, v, we have u v = u v. Calculate the inverse x for x = + i, calculate x y for x = 3 i, y = 3 + i 4. 6 Graphs and Nerves Consider the following digraph: Find a cycle of length in this digraph. Write the cycle as sequence x x... x of its arrows with the shown names, the cycle starting at x and ending at x. Which of the following graphs (they are the complete graphs with, 3, 4, and 5 vertexes) are having an Euler cycle? Use the criterium, which we have discussed in class (degree of a vertex). And also draw such a cycle, if it exists. We have seen that the nerve of the triadic covering C (3) = {I, II,..., V II} of the major scale C = {c, d, e, f, g, a, b} yields a Moebius strip, as shown to the left in the following figure. Show that if we replace the triad I by the seventh triad I 7+ in this covering, the Moebius strip is enriched by a tetrahedron, as shown in red color in figure??. How does the nerve of the covering C (4) = {I 7+, II 7,..., V II 7 } by the tetradic (i.e., seventh) degrees look like? Consider the two sets A = {a, b, c}, B = {x, y} of cardinality 3 and, respectively. How many digraph morphisms f : Loop(A) Loop(B) are there? How many morphisms f : Loop(A) [] into the directed -chain [] are there? How many f : [] Loop(A)? Give explicit lists of such morphisms. 7 Algebra and Matrixes Let us consider the so-called affine functions on the integers Z. They are determined by the selection of two integers t, m and denoted by T t m. By definition, such a function T t m : Z Z evaluates to T t m(x) = t + mx. These functions are central in music theory. In fact: If we interpret Z as the set of pitches (keys or MIDI pitches) T t is just the transposition of a pitch by t semitones, verify this! What is the musical meaning of the affine function T if 60 denotes middle c? Make an image! Denote by Aff(Z) the set of all affine functions on the integers. Show that this set defines a submonoid of the monoid Set(Z, Z) of all set functions f : Z Z, together with the monoid operation =, i.e., the compositions of set functions. First check the defining properties of a monoid for (Set(Z, Z),, Id Z ) and then also for this set Aff(Z). Show in particular, that the neutral element of Set(Z, Z) is an affine function. And then exhibit 6

7 the shape of the composition T t m T s n! To calculate this shape, take an argument x Z and calculate the resulting value (T t m T s n)(x). Next, do calculate the subgroup Aff(Z) of invertible elements of Aff(Z). Describe this group in terms of musical operations if we interpret Z as the set of pitches as above. Find out whether this group Aff(Z) is commutative or not. Consider the symmetric group S 8, i.e., the group of permutations of the set {,, 3,... 8} of natural numbers. Consider the permutations p = q = Calculate the product q p (attention: do not forget that the permutation to the right comes first, the one to the left second!). Consider the set p = {Id, p, p, p 3,...} of all powers of p. Show that this is a subgroup. What is its order (= cardinality?) Cycle decomposition of permutations: To do so, start with the cycle starting at. Then take the smallest number not contained in this cycle, an so forth, until all cycles are calculated. As a preliminary exercise, we calculate the cycle decomposition of q. The cycle of is C = (, 4,, 6, 5). The smallest number not in this first cycle is 3. The cycle of 3 is C = (3, 8, 7), so the total decomposition is q = C C. Now calculate the cycle decomposition of the permutation p. Consider the symmetric group S 4 and its element 3 4 r = 4 3 Write r as a product of the transpositions (, ),, 3), (, 4) (we know from the last lesson that this is possible). Hint: first multiply r by a transposition such that the product leaves 4 fixed. This can be done by prepending the transposition (, 4) to r, i.e., 3 4 (, 4) r = (, 4) = = (, ) 3 4 Then multiply that product by a transposition such that 3 remains fixed, etc. Then use the fact that transpositions are their own inverses. How? In our case, we have the even simpler situation that 7

8 (, 4) r = (, ) Therefore, multiplying the equation by (, 4) from the left we get i.e., since (, 4) (, 4) = Id, (, 4) (, 4) r = (, 4) (, ) r = (, 4) (, ) and we are done. Consider the set G = {x, y, z, u, v, w} of cardinality 6, and a multiplication : G G G given by the table X Y x y z u v w x u v w x y z y v w x y z u z w x y z u v u x y z u v w v y z u v w x w z u v w x y Is commutative? Is it associative? Is there a neutral element? Is this a monoid? Is it even a group? Exhibit inverses of its elements if possible. 7. Generators of Groups and Cyclic Groups. If we are given any subset X G of a group G, there is a unique smallest subgroup H G such that X H. There are two proofs of this fact. The first is quite abstract, but quite immediate: Take the set Σ of all subgroups K G such that X K. For example, G Σ. So Σ is not the empty set. Then consider the intersection S = Σ of all these subgroups. Evidently, S contains X as a subset since every element of Σ does so. But S is also a subgroup. Verify this! Then this intersection is the smallest subgroup of G that contains X. The second proof is more constructive and concrete. If this group exists, it must contain not only all elements x X, but also all elements of the following types:. the neutral element e G of the group G,. all products x x... x k, where the x i are either elements of X or inverses thereof. But these two types of elements are already a subgroup of G. Prove this! So this is the smallest subgroup of G containing X as a subset. This subgroup is denoted by X and called the subgroup of G generated by X. If the set is a singleton, i.e., contains just one element x: X = {x}, then we also write x instead of {x} and call this group a cyclic group. If x is an finite group, its order of order( x ) (recall, that this is the cardinality of the group) is called the order of x and denoted by order(x). If x is an infinite group, the order of x is also called infinite. 8

9 Example. Take the additive group of integers G = Z. Show that we have Z =, i.e., Z is cyclic. Can you find another generator x such that Z = x? Example. Show that every subgroup H of Z is cyclic. To do so, procede as follows: First, look at the trivial subgroup H = {0} = 0Z. Check that this is cyclic (which is its generator?). Then, take a non-trivial subgroup H Z. This one contains at least one positive integer h. Why? (Think of all possibilities and use the fact that H is a subgroup and therefore contains the inverse element for each of its elements.) Then, take the smallest positive integer m H. Now look at any element x H. By the division theorem we know that we may write x = a m + r, with a remainder 0 r < m. But then, since x and a m are both elements of H, we must have r H. As m is the minimal positive number in H, we must have r = 0. This shows that all elements of H are (positive or negative) multiples of m, i.e., we have H = m, the subgroup which we usually denote by mz. Example 3. The above results allow us to completely classify the cyclic groups, i.e., to give a complete description of such groups. In fact, suppose that a subgroup H of any group G is cyclic. This means that we have an element x G such that H = x. Consider now the group homomorphism f : Z G, which is defined by sending z Z to x z, more precisely: f(0) = e if z > 0, f(z) = x z (= x x x... x, z times) if z < 0, f(z) = (x ) z (= x x x... x, z times) For example, f(3) = x 3 = x x x and f( ) = x = (x ) = x x. Verify that this is a group homomorphism! By the theorem about kernels and images of group homomorphisms, which we have discussed in class, we know that we have a canonical isomorphism of groups Z/Ker(f) Im(f). But evidently, Im(f) = x. Therefore we know that Z/Ker(f) x. Using the classifiation of all subgroups of Z, we know that Ker(f) = mz for m = 0 or a positive m Z. This means that there is a (unique) integer m 0 such that Z m = Z/mZ x If m = 0, no power of x is the neutral element e G, and we have Z 0 = Z/0Z = Z x If m > 0, then x m = e is the smallest positive power of x that yiels e. Let us make a number of examples of cyclic groups! Take the element p = (, 3, 5, 6) S 6. What is the group p? Calculate the order of p and then describe the group generated by p as a quotient group of the integers! 9

10 Take the element i C (imaginary unit of the complex numbers) and describe the group i generated by i in the unit circle U = {z z = } (group operation = product of complex numbers). Show that a cyclic group is always commutative. conclude from this that the symmetric group S 3 is not cyclic. Use the Lagrange formula (for a finite group G and any subgroup H G, we have order(g) = (G : H) order(h)) to answer the following question: Is there an element p S 4 or order 7? Use the Lagrange formula to show that any group of prime order is cyclic. The group of pitch classes Z is evidently cyclic (why?). Find all generators x such that Z = x. Show that the soubgroup of the affine group GL(Z) = Aff(Z) generated by an inversion T t.( ) is isomorphic to Z. Consider the normal subgroup T Z of translations in GL(Z). Show that the quotient group GL(Z)/T Z is isomorphic to Z. In the set Z Z of notes (x, y), whose first coordinates are time (integer values), and whose second coordinates are pitch (integer values), consider the group C of permutations of the set Z Z generated by the inversion at zero I, i.e., I(x, y) = (x, y) and the retrograde R, i.e., R(x, y) = ( x, y). Show that C Z Z, the latter being the so-called Kleinian 4 group. Hint: Define a bijection C Z Z, which is a group isomorphism. 7. Matrixes and Affine Maps We have discussed matrixes and their operations. Let us first check by examples, whether we have understood these operations. Take the following six matrixes: K =, L = 5 3, M = , N = , t = 3, P = 4 Calculate the following matrixes (calcuate first, then compare to our results!). K + L. K L. 0

11 3. K 4. M N 5. N M 6. L 7. K 8. (affine maps!) T t.k(p ) And here are the results: 0. K + L = 6. K L = 3. K = 4. M N = 8 4 ( 4 ) 0 6 ( 5.5 ) N M = L does not exist, since det(l) = 0 7. K exists since det(k) = is different from zero. We have K = 3 det(k) = a b =. (Recall that for a matrix K = with non-vanishing 5 5 c d ( d b determinant, its inverse is K = det(k) 8. T t.k(p ) = t + K P = 4 c a ).)

12 x Next, we would like to know which vector Z = of the plane R y is mapped to the vector P = under the bijection of the plane defined by the matrix S =. So the problem is to find P such that P = S Z. Since S is invertible (check!), we can solve this equation by multiplying both sieds by S : S P = S S Z. This means Therefore we have Z = S P = Z. = 0. Given the -matrix R = ( ), we may define a map (denoted by the same x symbol R) R : R R via R(x, y) = R. Use the rules of matrix arithmetic to verify y that this is a group homomorphism of the additive group R onto the additive group R. Describe the image group Im(R) and the kernel Ker(R)! f Consider the digraph = a b, and the diagram D : GL(Z ) of affine g maps on Z, defined by D(f) = T.5, D(g) = T.3. Calculate all networks of this diagram. Recall for this that a network is a pair (x a, x b ) of elements of Z (one for each vertex of ) such that we have x b = D(f)(x a ) and x a = D(g)(x b ). Check that these are exactly the two networks (, 0) and (8, 6), and as we know from the class, this number of networks must be a divisor of.

I. GROUPS: BASIC DEFINITIONS AND EXAMPLES

I. GROUPS: BASIC DEFINITIONS AND EXAMPLES I GROUPS: BASIC DEFINITIONS AND EXAMPLES Definition 1: An operation on a set G is a function : G G G Definition 2: A group is a set G which is equipped with an operation and a special element e G, called

More information

Mathematics for Computer Science/Software Engineering. Notes for the course MSM1F3 Dr. R. A. Wilson

Mathematics for Computer Science/Software Engineering. Notes for the course MSM1F3 Dr. R. A. Wilson Mathematics for Computer Science/Software Engineering Notes for the course MSM1F3 Dr. R. A. Wilson October 1996 Chapter 1 Logic Lecture no. 1. We introduce the concept of a proposition, which is a statement

More information

Continued Fractions and the Euclidean Algorithm

Continued Fractions and the Euclidean Algorithm Continued Fractions and the Euclidean Algorithm Lecture notes prepared for MATH 326, Spring 997 Department of Mathematics and Statistics University at Albany William F Hammond Table of Contents Introduction

More information

Group Theory. Contents

Group Theory. Contents Group Theory Contents Chapter 1: Review... 2 Chapter 2: Permutation Groups and Group Actions... 3 Orbits and Transitivity... 6 Specific Actions The Right regular and coset actions... 8 The Conjugation

More information

INTRODUCTORY SET THEORY

INTRODUCTORY SET THEORY M.Sc. program in mathematics INTRODUCTORY SET THEORY Katalin Károlyi Department of Applied Analysis, Eötvös Loránd University H-1088 Budapest, Múzeum krt. 6-8. CONTENTS 1. SETS Set, equal sets, subset,

More information

3. Mathematical Induction

3. Mathematical Induction 3. MATHEMATICAL INDUCTION 83 3. Mathematical Induction 3.1. First Principle of Mathematical Induction. Let P (n) be a predicate with domain of discourse (over) the natural numbers N = {0, 1,,...}. If (1)

More information

Lecture 16 : Relations and Functions DRAFT

Lecture 16 : Relations and Functions DRAFT CS/Math 240: Introduction to Discrete Mathematics 3/29/2011 Lecture 16 : Relations and Functions Instructor: Dieter van Melkebeek Scribe: Dalibor Zelený DRAFT In Lecture 3, we described a correspondence

More information

Math Workshop October 2010 Fractions and Repeating Decimals

Math Workshop October 2010 Fractions and Repeating Decimals Math Workshop October 2010 Fractions and Repeating Decimals This evening we will investigate the patterns that arise when converting fractions to decimals. As an example of what we will be looking at,

More information

Introduction to Modern Algebra

Introduction to Modern Algebra Introduction to Modern Algebra David Joyce Clark University Version 0.0.6, 3 Oct 2008 1 1 Copyright (C) 2008. ii I dedicate this book to my friend and colleague Arthur Chou. Arthur encouraged me to write

More information

University of Lille I PC first year list of exercises n 7. Review

University of Lille I PC first year list of exercises n 7. Review University of Lille I PC first year list of exercises n 7 Review Exercise Solve the following systems in 4 different ways (by substitution, by the Gauss method, by inverting the matrix of coefficients

More information

Lemma 5.2. Let S be a set. (1) Let f and g be two permutations of S. Then the composition of f and g is a permutation of S.

Lemma 5.2. Let S be a set. (1) Let f and g be two permutations of S. Then the composition of f and g is a permutation of S. Definition 51 Let S be a set bijection f : S S 5 Permutation groups A permutation of S is simply a Lemma 52 Let S be a set (1) Let f and g be two permutations of S Then the composition of f and g is a

More information

EXERCISES FOR THE COURSE MATH 570, FALL 2010

EXERCISES FOR THE COURSE MATH 570, FALL 2010 EXERCISES FOR THE COURSE MATH 570, FALL 2010 EYAL Z. GOREN (1) Let G be a group and H Z(G) a subgroup such that G/H is cyclic. Prove that G is abelian. Conclude that every group of order p 2 (p a prime

More information

Cartesian Products and Relations

Cartesian Products and Relations Cartesian Products and Relations Definition (Cartesian product) If A and B are sets, the Cartesian product of A and B is the set A B = {(a, b) :(a A) and (b B)}. The following points are worth special

More information

8 Divisibility and prime numbers

8 Divisibility and prime numbers 8 Divisibility and prime numbers 8.1 Divisibility In this short section we extend the concept of a multiple from the natural numbers to the integers. We also summarize several other terms that express

More information

Mathematics Course 111: Algebra I Part IV: Vector Spaces

Mathematics Course 111: Algebra I Part IV: Vector Spaces Mathematics Course 111: Algebra I Part IV: Vector Spaces D. R. Wilkins Academic Year 1996-7 9 Vector Spaces A vector space over some field K is an algebraic structure consisting of a set V on which are

More information

Chapter 4, Arithmetic in F [x] Polynomial arithmetic and the division algorithm.

Chapter 4, Arithmetic in F [x] Polynomial arithmetic and the division algorithm. Chapter 4, Arithmetic in F [x] Polynomial arithmetic and the division algorithm. We begin by defining the ring of polynomials with coefficients in a ring R. After some preliminary results, we specialize

More information

= 2 + 1 2 2 = 3 4, Now assume that P (k) is true for some fixed k 2. This means that

= 2 + 1 2 2 = 3 4, Now assume that P (k) is true for some fixed k 2. This means that Instructions. Answer each of the questions on your own paper, and be sure to show your work so that partial credit can be adequately assessed. Credit will not be given for answers (even correct ones) without

More information

ABSTRACT ALGEBRA: A STUDY GUIDE FOR BEGINNERS

ABSTRACT ALGEBRA: A STUDY GUIDE FOR BEGINNERS ABSTRACT ALGEBRA: A STUDY GUIDE FOR BEGINNERS John A. Beachy Northern Illinois University 2014 ii J.A.Beachy This is a supplement to Abstract Algebra, Third Edition by John A. Beachy and William D. Blair

More information

Mathematical Induction. Lecture 10-11

Mathematical Induction. Lecture 10-11 Mathematical Induction Lecture 10-11 Menu Mathematical Induction Strong Induction Recursive Definitions Structural Induction Climbing an Infinite Ladder Suppose we have an infinite ladder: 1. We can reach

More information

This chapter is all about cardinality of sets. At first this looks like a

This chapter is all about cardinality of sets. At first this looks like a CHAPTER Cardinality of Sets This chapter is all about cardinality of sets At first this looks like a very simple concept To find the cardinality of a set, just count its elements If A = { a, b, c, d },

More information

Handout #1: Mathematical Reasoning

Handout #1: Mathematical Reasoning Math 101 Rumbos Spring 2010 1 Handout #1: Mathematical Reasoning 1 Propositional Logic A proposition is a mathematical statement that it is either true or false; that is, a statement whose certainty or

More information

1 Sets and Set Notation.

1 Sets and Set Notation. LINEAR ALGEBRA MATH 27.6 SPRING 23 (COHEN) LECTURE NOTES Sets and Set Notation. Definition (Naive Definition of a Set). A set is any collection of objects, called the elements of that set. We will most

More information

Math Review. for the Quantitative Reasoning Measure of the GRE revised General Test

Math Review. for the Quantitative Reasoning Measure of the GRE revised General Test Math Review for the Quantitative Reasoning Measure of the GRE revised General Test www.ets.org Overview This Math Review will familiarize you with the mathematical skills and concepts that are important

More information

Mathematics Review for MS Finance Students

Mathematics Review for MS Finance Students Mathematics Review for MS Finance Students Anthony M. Marino Department of Finance and Business Economics Marshall School of Business Lecture 1: Introductory Material Sets The Real Number System Functions,

More information

Sample Induction Proofs

Sample Induction Proofs Math 3 Worksheet: Induction Proofs III, Sample Proofs A.J. Hildebrand Sample Induction Proofs Below are model solutions to some of the practice problems on the induction worksheets. The solutions given

More information

8 Primes and Modular Arithmetic

8 Primes and Modular Arithmetic 8 Primes and Modular Arithmetic 8.1 Primes and Factors Over two millennia ago already, people all over the world were considering the properties of numbers. One of the simplest concepts is prime numbers.

More information

A Second Course in Mathematics Concepts for Elementary Teachers: Theory, Problems, and Solutions

A Second Course in Mathematics Concepts for Elementary Teachers: Theory, Problems, and Solutions A Second Course in Mathematics Concepts for Elementary Teachers: Theory, Problems, and Solutions Marcel B. Finan Arkansas Tech University c All Rights Reserved First Draft February 8, 2006 1 Contents 25

More information

CS 103X: Discrete Structures Homework Assignment 3 Solutions

CS 103X: Discrete Structures Homework Assignment 3 Solutions CS 103X: Discrete Structures Homework Assignment 3 s Exercise 1 (20 points). On well-ordering and induction: (a) Prove the induction principle from the well-ordering principle. (b) Prove the well-ordering

More information

Chapter 3. Cartesian Products and Relations. 3.1 Cartesian Products

Chapter 3. Cartesian Products and Relations. 3.1 Cartesian Products Chapter 3 Cartesian Products and Relations The material in this chapter is the first real encounter with abstraction. Relations are very general thing they are a special type of subset. After introducing

More information

Course Syllabus. MATH 1350-Mathematics for Teachers I. Revision Date: 8/15/2016

Course Syllabus. MATH 1350-Mathematics for Teachers I. Revision Date: 8/15/2016 Course Syllabus MATH 1350-Mathematics for Teachers I Revision Date: 8/15/2016 Catalog Description: This course is intended to build or reinforce a foundation in fundamental mathematics concepts and skills.

More information

a 11 x 1 + a 12 x 2 + + a 1n x n = b 1 a 21 x 1 + a 22 x 2 + + a 2n x n = b 2.

a 11 x 1 + a 12 x 2 + + a 1n x n = b 1 a 21 x 1 + a 22 x 2 + + a 2n x n = b 2. Chapter 1 LINEAR EQUATIONS 1.1 Introduction to linear equations A linear equation in n unknowns x 1, x,, x n is an equation of the form a 1 x 1 + a x + + a n x n = b, where a 1, a,..., a n, b are given

More information

Copy in your notebook: Add an example of each term with the symbols used in algebra 2 if there are any.

Copy in your notebook: Add an example of each term with the symbols used in algebra 2 if there are any. Algebra 2 - Chapter Prerequisites Vocabulary Copy in your notebook: Add an example of each term with the symbols used in algebra 2 if there are any. P1 p. 1 1. counting(natural) numbers - {1,2,3,4,...}

More information

Answer Key for California State Standards: Algebra I

Answer Key for California State Standards: Algebra I Algebra I: Symbolic reasoning and calculations with symbols are central in algebra. Through the study of algebra, a student develops an understanding of the symbolic language of mathematics and the sciences.

More information

6.2 Permutations continued

6.2 Permutations continued 6.2 Permutations continued Theorem A permutation on a finite set A is either a cycle or can be expressed as a product (composition of disjoint cycles. Proof is by (strong induction on the number, r, of

More information

Math 3000 Section 003 Intro to Abstract Math Homework 2

Math 3000 Section 003 Intro to Abstract Math Homework 2 Math 3000 Section 003 Intro to Abstract Math Homework 2 Department of Mathematical and Statistical Sciences University of Colorado Denver, Spring 2012 Solutions (February 13, 2012) Please note that these

More information

Examples of Functions

Examples of Functions Examples of Functions In this document is provided examples of a variety of functions. The purpose is to convince the beginning student that functions are something quite different than polynomial equations.

More information

Lecture 13 - Basic Number Theory.

Lecture 13 - Basic Number Theory. Lecture 13 - Basic Number Theory. Boaz Barak March 22, 2010 Divisibility and primes Unless mentioned otherwise throughout this lecture all numbers are non-negative integers. We say that A divides B, denoted

More information

26 Integers: Multiplication, Division, and Order

26 Integers: Multiplication, Division, and Order 26 Integers: Multiplication, Division, and Order Integer multiplication and division are extensions of whole number multiplication and division. In multiplying and dividing integers, the one new issue

More information

How To Prove The Dirichlet Unit Theorem

How To Prove The Dirichlet Unit Theorem Chapter 6 The Dirichlet Unit Theorem As usual, we will be working in the ring B of algebraic integers of a number field L. Two factorizations of an element of B are regarded as essentially the same if

More information

Introduction. Appendix D Mathematical Induction D1

Introduction. Appendix D Mathematical Induction D1 Appendix D Mathematical Induction D D Mathematical Induction Use mathematical induction to prove a formula. Find a sum of powers of integers. Find a formula for a finite sum. Use finite differences to

More information

GENERATING SETS KEITH CONRAD

GENERATING SETS KEITH CONRAD GENERATING SETS KEITH CONRAD 1 Introduction In R n, every vector can be written as a unique linear combination of the standard basis e 1,, e n A notion weaker than a basis is a spanning set: a set of vectors

More information

How To Understand The Theory Of Hyperreals

How To Understand The Theory Of Hyperreals Ultraproducts and Applications I Brent Cody Virginia Commonwealth University September 2, 2013 Outline Background of the Hyperreals Filters and Ultrafilters Construction of the Hyperreals The Transfer

More information

Chapter 7. Permutation Groups

Chapter 7. Permutation Groups Chapter 7 Permutation Groups () We started the study of groups by considering planar isometries In the previous chapter, we learnt that finite groups of planar isometries can only be cyclic or dihedral

More information

CONTENTS. Please note:

CONTENTS. Please note: CONTENTS Introduction...iv. Number Systems... 2. Algebraic Expressions.... Factorising...24 4. Solving Linear Equations...8. Solving Quadratic Equations...0 6. Simultaneous Equations.... Long Division

More information

it is easy to see that α = a

it is easy to see that α = a 21. Polynomial rings Let us now turn out attention to determining the prime elements of a polynomial ring, where the coefficient ring is a field. We already know that such a polynomial ring is a UF. Therefore

More information

Module MA3411: Abstract Algebra Galois Theory Appendix Michaelmas Term 2013

Module MA3411: Abstract Algebra Galois Theory Appendix Michaelmas Term 2013 Module MA3411: Abstract Algebra Galois Theory Appendix Michaelmas Term 2013 D. R. Wilkins Copyright c David R. Wilkins 1997 2013 Contents A Cyclotomic Polynomials 79 A.1 Minimum Polynomials of Roots of

More information

SECTION 10-2 Mathematical Induction

SECTION 10-2 Mathematical Induction 73 0 Sequences and Series 6. Approximate e 0. using the first five terms of the series. Compare this approximation with your calculator evaluation of e 0.. 6. Approximate e 0.5 using the first five terms

More information

FUNCTIONAL ANALYSIS LECTURE NOTES: QUOTIENT SPACES

FUNCTIONAL ANALYSIS LECTURE NOTES: QUOTIENT SPACES FUNCTIONAL ANALYSIS LECTURE NOTES: QUOTIENT SPACES CHRISTOPHER HEIL 1. Cosets and the Quotient Space Any vector space is an abelian group under the operation of vector addition. So, if you are have studied

More information

CHAPTER SIX IRREDUCIBILITY AND FACTORIZATION 1. BASIC DIVISIBILITY THEORY

CHAPTER SIX IRREDUCIBILITY AND FACTORIZATION 1. BASIC DIVISIBILITY THEORY January 10, 2010 CHAPTER SIX IRREDUCIBILITY AND FACTORIZATION 1. BASIC DIVISIBILITY THEORY The set of polynomials over a field F is a ring, whose structure shares with the ring of integers many characteristics.

More information

CHAPTER 5. Number Theory. 1. Integers and Division. Discussion

CHAPTER 5. Number Theory. 1. Integers and Division. Discussion CHAPTER 5 Number Theory 1. Integers and Division 1.1. Divisibility. Definition 1.1.1. Given two integers a and b we say a divides b if there is an integer c such that b = ac. If a divides b, we write a

More information

Solve addition and subtraction word problems, and add and subtract within 10, e.g., by using objects or drawings to represent the problem.

Solve addition and subtraction word problems, and add and subtract within 10, e.g., by using objects or drawings to represent the problem. Solve addition and subtraction word problems, and add and subtract within 10, e.g., by using objects or drawings to represent the problem. Solve word problems that call for addition of three whole numbers

More information

This asserts two sets are equal iff they have the same elements, that is, a set is determined by its elements.

This asserts two sets are equal iff they have the same elements, that is, a set is determined by its elements. 3. Axioms of Set theory Before presenting the axioms of set theory, we first make a few basic comments about the relevant first order logic. We will give a somewhat more detailed discussion later, but

More information

You know from calculus that functions play a fundamental role in mathematics.

You know from calculus that functions play a fundamental role in mathematics. CHPTER 12 Functions You know from calculus that functions play a fundamental role in mathematics. You likely view a function as a kind of formula that describes a relationship between two (or more) quantities.

More information

Continued Fractions. Darren C. Collins

Continued Fractions. Darren C. Collins Continued Fractions Darren C Collins Abstract In this paper, we discuss continued fractions First, we discuss the definition and notation Second, we discuss the development of the subject throughout history

More information

GROUPS ACTING ON A SET

GROUPS ACTING ON A SET GROUPS ACTING ON A SET MATH 435 SPRING 2012 NOTES FROM FEBRUARY 27TH, 2012 1. Left group actions Definition 1.1. Suppose that G is a group and S is a set. A left (group) action of G on S is a rule for

More information

MATH10212 Linear Algebra. Systems of Linear Equations. Definition. An n-dimensional vector is a row or a column of n numbers (or letters): a 1.

MATH10212 Linear Algebra. Systems of Linear Equations. Definition. An n-dimensional vector is a row or a column of n numbers (or letters): a 1. MATH10212 Linear Algebra Textbook: D. Poole, Linear Algebra: A Modern Introduction. Thompson, 2006. ISBN 0-534-40596-7. Systems of Linear Equations Definition. An n-dimensional vector is a row or a column

More information

Homework until Test #2

Homework until Test #2 MATH31: Number Theory Homework until Test # Philipp BRAUN Section 3.1 page 43, 1. It has been conjectured that there are infinitely many primes of the form n. Exhibit five such primes. Solution. Five such

More information

MATH10040 Chapter 2: Prime and relatively prime numbers

MATH10040 Chapter 2: Prime and relatively prime numbers MATH10040 Chapter 2: Prime and relatively prime numbers Recall the basic definition: 1. Prime numbers Definition 1.1. Recall that a positive integer is said to be prime if it has precisely two positive

More information

A Little Set Theory (Never Hurt Anybody)

A Little Set Theory (Never Hurt Anybody) A Little Set Theory (Never Hurt Anybody) Matthew Saltzman Department of Mathematical Sciences Clemson University Draft: August 21, 2013 1 Introduction The fundamental ideas of set theory and the algebra

More information

Chapter 13: Basic ring theory

Chapter 13: Basic ring theory Chapter 3: Basic ring theory Matthew Macauley Department of Mathematical Sciences Clemson University http://www.math.clemson.edu/~macaule/ Math 42, Spring 24 M. Macauley (Clemson) Chapter 3: Basic ring

More information

Precalculus REVERSE CORRELATION. Content Expectations for. Precalculus. Michigan CONTENT EXPECTATIONS FOR PRECALCULUS CHAPTER/LESSON TITLES

Precalculus REVERSE CORRELATION. Content Expectations for. Precalculus. Michigan CONTENT EXPECTATIONS FOR PRECALCULUS CHAPTER/LESSON TITLES Content Expectations for Precalculus Michigan Precalculus 2011 REVERSE CORRELATION CHAPTER/LESSON TITLES Chapter 0 Preparing for Precalculus 0-1 Sets There are no state-mandated Precalculus 0-2 Operations

More information

PUTNAM TRAINING POLYNOMIALS. Exercises 1. Find a polynomial with integral coefficients whose zeros include 2 + 5.

PUTNAM TRAINING POLYNOMIALS. Exercises 1. Find a polynomial with integral coefficients whose zeros include 2 + 5. PUTNAM TRAINING POLYNOMIALS (Last updated: November 17, 2015) Remark. This is a list of exercises on polynomials. Miguel A. Lerma Exercises 1. Find a polynomial with integral coefficients whose zeros include

More information

Overview. Essential Questions. Precalculus, Quarter 4, Unit 4.5 Build Arithmetic and Geometric Sequences and Series

Overview. Essential Questions. Precalculus, Quarter 4, Unit 4.5 Build Arithmetic and Geometric Sequences and Series Sequences and Series Overview Number of instruction days: 4 6 (1 day = 53 minutes) Content to Be Learned Write arithmetic and geometric sequences both recursively and with an explicit formula, use them

More information

Undergraduate Notes in Mathematics. Arkansas Tech University Department of Mathematics

Undergraduate Notes in Mathematics. Arkansas Tech University Department of Mathematics Undergraduate Notes in Mathematics Arkansas Tech University Department of Mathematics An Introductory Single Variable Real Analysis: A Learning Approach through Problem Solving Marcel B. Finan c All Rights

More information

Notes on Algebraic Structures. Peter J. Cameron

Notes on Algebraic Structures. Peter J. Cameron Notes on Algebraic Structures Peter J. Cameron ii Preface These are the notes of the second-year course Algebraic Structures I at Queen Mary, University of London, as I taught it in the second semester

More information

(0, 0) : order 1; (0, 1) : order 4; (0, 2) : order 2; (0, 3) : order 4; (1, 0) : order 2; (1, 1) : order 4; (1, 2) : order 2; (1, 3) : order 4.

(0, 0) : order 1; (0, 1) : order 4; (0, 2) : order 2; (0, 3) : order 4; (1, 0) : order 2; (1, 1) : order 4; (1, 2) : order 2; (1, 3) : order 4. 11.01 List the elements of Z 2 Z 4. Find the order of each of the elements is this group cyclic? Solution: The elements of Z 2 Z 4 are: (0, 0) : order 1; (0, 1) : order 4; (0, 2) : order 2; (0, 3) : order

More information

COMMUTATIVITY DEGREES OF WREATH PRODUCTS OF FINITE ABELIAN GROUPS

COMMUTATIVITY DEGREES OF WREATH PRODUCTS OF FINITE ABELIAN GROUPS COMMUTATIVITY DEGREES OF WREATH PRODUCTS OF FINITE ABELIAN GROUPS IGOR V. EROVENKO AND B. SURY ABSTRACT. We compute commutativity degrees of wreath products A B of finite abelian groups A and B. When B

More information

Linear Algebra I. Ronald van Luijk, 2012

Linear Algebra I. Ronald van Luijk, 2012 Linear Algebra I Ronald van Luijk, 2012 With many parts from Linear Algebra I by Michael Stoll, 2007 Contents 1. Vector spaces 3 1.1. Examples 3 1.2. Fields 4 1.3. The field of complex numbers. 6 1.4.

More information

Application. Outline. 3-1 Polynomial Functions 3-2 Finding Rational Zeros of. Polynomial. 3-3 Approximating Real Zeros of.

Application. Outline. 3-1 Polynomial Functions 3-2 Finding Rational Zeros of. Polynomial. 3-3 Approximating Real Zeros of. Polynomial and Rational Functions Outline 3-1 Polynomial Functions 3-2 Finding Rational Zeros of Polynomials 3-3 Approximating Real Zeros of Polynomials 3-4 Rational Functions Chapter 3 Group Activity:

More information

MATHEMATICAL INDUCTION. Mathematical Induction. This is a powerful method to prove properties of positive integers.

MATHEMATICAL INDUCTION. Mathematical Induction. This is a powerful method to prove properties of positive integers. MATHEMATICAL INDUCTION MIGUEL A LERMA (Last updated: February 8, 003) Mathematical Induction This is a powerful method to prove properties of positive integers Principle of Mathematical Induction Let P

More information

CHAPTER 3. Methods of Proofs. 1. Logical Arguments and Formal Proofs

CHAPTER 3. Methods of Proofs. 1. Logical Arguments and Formal Proofs CHAPTER 3 Methods of Proofs 1. Logical Arguments and Formal Proofs 1.1. Basic Terminology. An axiom is a statement that is given to be true. A rule of inference is a logical rule that is used to deduce

More information

Vocabulary Words and Definitions for Algebra

Vocabulary Words and Definitions for Algebra Name: Period: Vocabulary Words and s for Algebra Absolute Value Additive Inverse Algebraic Expression Ascending Order Associative Property Axis of Symmetry Base Binomial Coefficient Combine Like Terms

More information

Ideal Class Group and Units

Ideal Class Group and Units Chapter 4 Ideal Class Group and Units We are now interested in understanding two aspects of ring of integers of number fields: how principal they are (that is, what is the proportion of principal ideals

More information

Just the Factors, Ma am

Just the Factors, Ma am 1 Introduction Just the Factors, Ma am The purpose of this note is to find and study a method for determining and counting all the positive integer divisors of a positive integer Let N be a given positive

More information

Estimated Pre Calculus Pacing Timeline

Estimated Pre Calculus Pacing Timeline Estimated Pre Calculus Pacing Timeline 2010-2011 School Year The timeframes listed on this calendar are estimates based on a fifty-minute class period. You may need to adjust some of them from time to

More information

Prentice Hall: Middle School Math, Course 1 2002 Correlated to: New York Mathematics Learning Standards (Intermediate)

Prentice Hall: Middle School Math, Course 1 2002 Correlated to: New York Mathematics Learning Standards (Intermediate) New York Mathematics Learning Standards (Intermediate) Mathematical Reasoning Key Idea: Students use MATHEMATICAL REASONING to analyze mathematical situations, make conjectures, gather evidence, and construct

More information

Basic Concepts of Point Set Topology Notes for OU course Math 4853 Spring 2011

Basic Concepts of Point Set Topology Notes for OU course Math 4853 Spring 2011 Basic Concepts of Point Set Topology Notes for OU course Math 4853 Spring 2011 A. Miller 1. Introduction. The definitions of metric space and topological space were developed in the early 1900 s, largely

More information

ON GALOIS REALIZATIONS OF THE 2-COVERABLE SYMMETRIC AND ALTERNATING GROUPS

ON GALOIS REALIZATIONS OF THE 2-COVERABLE SYMMETRIC AND ALTERNATING GROUPS ON GALOIS REALIZATIONS OF THE 2-COVERABLE SYMMETRIC AND ALTERNATING GROUPS DANIEL RABAYEV AND JACK SONN Abstract. Let f(x) be a monic polynomial in Z[x] with no rational roots but with roots in Q p for

More information

MATRIX ALGEBRA AND SYSTEMS OF EQUATIONS

MATRIX ALGEBRA AND SYSTEMS OF EQUATIONS MATRIX ALGEBRA AND SYSTEMS OF EQUATIONS Systems of Equations and Matrices Representation of a linear system The general system of m equations in n unknowns can be written a x + a 2 x 2 + + a n x n b a

More information

So let us begin our quest to find the holy grail of real analysis.

So let us begin our quest to find the holy grail of real analysis. 1 Section 5.2 The Complete Ordered Field: Purpose of Section We present an axiomatic description of the real numbers as a complete ordered field. The axioms which describe the arithmetic of the real numbers

More information

7. Some irreducible polynomials

7. Some irreducible polynomials 7. Some irreducible polynomials 7.1 Irreducibles over a finite field 7.2 Worked examples Linear factors x α of a polynomial P (x) with coefficients in a field k correspond precisely to roots α k [1] of

More information

PYTHAGOREAN TRIPLES KEITH CONRAD

PYTHAGOREAN TRIPLES KEITH CONRAD PYTHAGOREAN TRIPLES KEITH CONRAD 1. Introduction A Pythagorean triple is a triple of positive integers (a, b, c) where a + b = c. Examples include (3, 4, 5), (5, 1, 13), and (8, 15, 17). Below is an ancient

More information

Math 223 Abstract Algebra Lecture Notes

Math 223 Abstract Algebra Lecture Notes Math 223 Abstract Algebra Lecture Notes Steven Tschantz Spring 2001 (Apr. 23 version) Preamble These notes are intended to supplement the lectures and make up for the lack of a textbook for the course

More information

MATRIX ALGEBRA AND SYSTEMS OF EQUATIONS. + + x 2. x n. a 11 a 12 a 1n b 1 a 21 a 22 a 2n b 2 a 31 a 32 a 3n b 3. a m1 a m2 a mn b m

MATRIX ALGEBRA AND SYSTEMS OF EQUATIONS. + + x 2. x n. a 11 a 12 a 1n b 1 a 21 a 22 a 2n b 2 a 31 a 32 a 3n b 3. a m1 a m2 a mn b m MATRIX ALGEBRA AND SYSTEMS OF EQUATIONS 1. SYSTEMS OF EQUATIONS AND MATRICES 1.1. Representation of a linear system. The general system of m equations in n unknowns can be written a 11 x 1 + a 12 x 2 +

More information

(a) Write each of p and q as a polynomial in x with coefficients in Z[y, z]. deg(p) = 7 deg(q) = 9

(a) Write each of p and q as a polynomial in x with coefficients in Z[y, z]. deg(p) = 7 deg(q) = 9 Homework #01, due 1/20/10 = 9.1.2, 9.1.4, 9.1.6, 9.1.8, 9.2.3 Additional problems for study: 9.1.1, 9.1.3, 9.1.5, 9.1.13, 9.2.1, 9.2.2, 9.2.4, 9.2.5, 9.2.6, 9.3.2, 9.3.3 9.1.1 (This problem was not assigned

More information

Lecture 17 : Equivalence and Order Relations DRAFT

Lecture 17 : Equivalence and Order Relations DRAFT CS/Math 240: Introduction to Discrete Mathematics 3/31/2011 Lecture 17 : Equivalence and Order Relations Instructor: Dieter van Melkebeek Scribe: Dalibor Zelený DRAFT Last lecture we introduced the notion

More information

1 Homework 1. [p 0 q i+j +... + p i 1 q j+1 ] + [p i q j ] + [p i+1 q j 1 +... + p i+j q 0 ]

1 Homework 1. [p 0 q i+j +... + p i 1 q j+1 ] + [p i q j ] + [p i+1 q j 1 +... + p i+j q 0 ] 1 Homework 1 (1) Prove the ideal (3,x) is a maximal ideal in Z[x]. SOLUTION: Suppose we expand this ideal by including another generator polynomial, P / (3, x). Write P = n + x Q with n an integer not

More information

Group Fundamentals. Chapter 1. 1.1 Groups and Subgroups. 1.1.1 Definition

Group Fundamentals. Chapter 1. 1.1 Groups and Subgroups. 1.1.1 Definition Chapter 1 Group Fundamentals 1.1 Groups and Subgroups 1.1.1 Definition A group is a nonempty set G on which there is defined a binary operation (a, b) ab satisfying the following properties. Closure: If

More information

U.C. Berkeley CS276: Cryptography Handout 0.1 Luca Trevisan January, 2009. Notes on Algebra

U.C. Berkeley CS276: Cryptography Handout 0.1 Luca Trevisan January, 2009. Notes on Algebra U.C. Berkeley CS276: Cryptography Handout 0.1 Luca Trevisan January, 2009 Notes on Algebra These notes contain as little theory as possible, and most results are stated without proof. Any introductory

More information

Properties of sequences Since a sequence is a special kind of function it has analogous properties to functions:

Properties of sequences Since a sequence is a special kind of function it has analogous properties to functions: Sequences and Series A sequence is a special kind of function whose domain is N - the set of natural numbers. The range of a sequence is the collection of terms that make up the sequence. Just as the word

More information

To define function and introduce operations on the set of functions. To investigate which of the field properties hold in the set of functions

To define function and introduce operations on the set of functions. To investigate which of the field properties hold in the set of functions Chapter 7 Functions This unit defines and investigates functions as algebraic objects. First, we define functions and discuss various means of representing them. Then we introduce operations on functions

More information

Notes on Determinant

Notes on Determinant ENGG2012B Advanced Engineering Mathematics Notes on Determinant Lecturer: Kenneth Shum Lecture 9-18/02/2013 The determinant of a system of linear equations determines whether the solution is unique, without

More information

CONSEQUENCES OF THE SYLOW THEOREMS

CONSEQUENCES OF THE SYLOW THEOREMS CONSEQUENCES OF THE SYLOW THEOREMS KEITH CONRAD For a group theorist, Sylow s Theorem is such a basic tool, and so fundamental, that it is used almost without thinking, like breathing. Geoff Robinson 1.

More information

Inner Product Spaces

Inner Product Spaces Math 571 Inner Product Spaces 1. Preliminaries An inner product space is a vector space V along with a function, called an inner product which associates each pair of vectors u, v with a scalar u, v, and

More information

MA651 Topology. Lecture 6. Separation Axioms.

MA651 Topology. Lecture 6. Separation Axioms. MA651 Topology. Lecture 6. Separation Axioms. This text is based on the following books: Fundamental concepts of topology by Peter O Neil Elements of Mathematics: General Topology by Nicolas Bourbaki Counterexamples

More information

MATH 60 NOTEBOOK CERTIFICATIONS

MATH 60 NOTEBOOK CERTIFICATIONS MATH 60 NOTEBOOK CERTIFICATIONS Chapter #1: Integers and Real Numbers 1.1a 1.1b 1.2 1.3 1.4 1.8 Chapter #2: Algebraic Expressions, Linear Equations, and Applications 2.1a 2.1b 2.1c 2.2 2.3a 2.3b 2.4 2.5

More information

Discrete Mathematics and Probability Theory Fall 2009 Satish Rao, David Tse Note 2

Discrete Mathematics and Probability Theory Fall 2009 Satish Rao, David Tse Note 2 CS 70 Discrete Mathematics and Probability Theory Fall 2009 Satish Rao, David Tse Note 2 Proofs Intuitively, the concept of proof should already be familiar We all like to assert things, and few of us

More information

Math 4310 Handout - Quotient Vector Spaces

Math 4310 Handout - Quotient Vector Spaces Math 4310 Handout - Quotient Vector Spaces Dan Collins The textbook defines a subspace of a vector space in Chapter 4, but it avoids ever discussing the notion of a quotient space. This is understandable

More information

Discrete Mathematics. Hans Cuypers. October 11, 2007

Discrete Mathematics. Hans Cuypers. October 11, 2007 Hans Cuypers October 11, 2007 1 Contents 1. Relations 4 1.1. Binary relations................................ 4 1.2. Equivalence relations............................. 6 1.3. Relations and Directed Graphs.......................

More information

α = u v. In other words, Orthogonal Projection

α = u v. In other words, Orthogonal Projection Orthogonal Projection Given any nonzero vector v, it is possible to decompose an arbitrary vector u into a component that points in the direction of v and one that points in a direction orthogonal to v

More information