Integral Domains

Total Page:16

File Type:pdf, Size:1020Kb

Integral Domains Integral Domains 1. Localization The intent of this section is to make formal the process of forming the rationals Q from the integers Z. This process, known as localization, is applicable to a large class of rings. We will define Q(x), the ring of rational functions in one variable (over Q), using this process. Another goal here is to extend notions of divisibility and factorization in Z to integral domains. One can associate any rational number p=q 2 Q with the ordered pair (p; q) 2 Z×Znf0g. This is not a bijection of sets, however, because 1=2 = 2=4 but (1; 2) 6= (2; 4). Thus, we place an equivalence relation on the latter set. Recall that a=b = c=d if and only if ad = bc. Hence, we say (a; b) ∼ (c; d)) if ad = bc. Lemma 1. Let D be any integral domain and define the set S = f(a; b): a; b 2 D and b 6= 0g: The relation ∼ on S given by (a; b) ∼ (c; d) if ad = bc is an equivalence relation. Proof. Let (a; b) 2 S. Then ab = ba because D is an integral domain (and hence commutative). Thus, (a; b) ∼ (a; b) and so ∼ is reflexive. Let (a; b); (c; d) 2 S such that (a; b) ∼ (c; d). Then ad = bc and so cb = da because D is an integral domain. Thus, (c; d) ∼ (a; b) and so ∼ is symmetric. Finally, suppose (a; b) ∼ (c; d) and (c; d) ∼ (e; f) in S. Then ad = bc and cf = de. Since D is an integral domain without zero divisors, then ade = bce so acf = bce. Thus, af = be so (a; b) ∼ (e; f) and ∼ is transitive. Let [a; b] denote the equivalence class of (a; b) 2 S under ∼. The set of such equivalence classes is denoted FD. We will prove that FD is in fact a field, justifying the name field of fractions of D. The operations on FD are defined to mimic the operations of adding and multiplying fractions. For [a; b]; [c; d] 2 FD, define [a; b] + [c; d] = [ad + bc; bd] and [a; b] · [c; d] = [ac; bd]: Lemma 2. The operations of addition and multiplication above are binary operations on FD. These notes are derived primarily from Abstract Algebra, Theory and Applications by Thomas Judson (16ed). Most of this material is drawn from Chapter 18. Hungerford's Algebra was also consulted. Last Updated: December 6, 2019 1 Proof. That FD is closed under these operations is clear. We need only show that they are well- defined (independent of equivalence class). Let [a1; b1]; [a2; b2]; [c1; d1]; [c2; d2] 2 FD with [a1; b1] = [a2; b2] and [c1; d1] = [c2; d2]. Thus, a1b2 = b1a2 and c1d2 = d1c2. We claim [a1; b1] + [c1; d1] = [a2; b2] + [c2; d2]. Equivalently, [a1d1 + b1c1; b1d1] = [a2d2 + b2c2; b2d2] or (a1d1 + b1c1)(b2d2) = (b1d1)(a2d2 + b2c2): We have (a1d1 + b1c1)(b2d2) = (a1d1)(b2d2) + (b1c1)(b2d2) = (a1b2)(d1d2) + (b1b2)(c1d2) = (b1a2)(d1d2) + (b1b2)(d1c2) = (b1d1)(a2d2 + b2c2): Checking the operation of multiplication is left as an (easier) exercise. Lemma 3. The set FD with the above binary operations is a field. Proof. We claim the additive identity is [0; 1]. Let [a; b] 2 FD, then [a; b] + [0; 1] = [a · 1 + b · 0; b · 1] = [a; b]: Associativity is left as an exercise. We claim the additive inverse of [a; b] is [−a; b] (note −a 2 D because D is a ring). One checks that [a; b] + [−a; b] = [ab + b(−a); b2] = [0; b2] = [0; 1]. (Note that 2 this last equality follows because 0 · 1 = b · 0.) Thus, (FD; +) is an abelian group. Associativity and commutivity of multiplication are left as an exercise. We check the left distributive property. Let [a; b]; [c; d]; [e; f] 2 FD. Then [a; b][c; d] + [a; b][e; f] = [ac; bd] + [ae; bf] = [acbf + bdae; bdbf] = [acf + dae; bdf] = [a; b][cf + de; df] = [a; b]([c; d] + [e; f]): By commutivity, the right distributive property also holds. Hence, FD is a commutative ring. The multiplicative identity in FD is [1; 1]. This is an easy check: [a; b][1; 1] = [a; b]. Moreover, the multiplicative inverse of [a; b] is [b; a] as [a; b][b; a] = [ab; ba] = [1; 1]. Thus, FD a field. Definition 1. The field FD defined above is the field of fractions of D. We next aim to show that, in some sense, FD is the smallest field containing D. Lemma 4. Let D be an integral domain and FD its field of fractions. There is an injective homomorphism φ : D ! FD defined by φ(a) = [a; 1]. 2 Proof. Let a; b 2 D, then φ(a) + φ(b) = [a; 1] + [b; 1] = [a + b; 1] = φ(a + b) φ(a)φ(b) = [a; 1][b; 1] = [ab; 1] = φ(ab): Thus, φ is a ring homomorphism. Now suppose φ(a) = 0, then [a; 1] = [0; 1], so a = 0. Thus, ker φ = f0g and φ is injective. As a consequence of this lemma, D is isomorphic to a subring of FD. The next theorem is an example of a universal property. Theorem 5. Let D be an integral domain and FD its field of fractions. If E is any field containing D, then there exists a unique injective homomorphism : FD ! E such that (φ(a)) = a for all a 2 D. −1 Proof. Let E be any field containing D. Define a map : Fd ! E by [a; b] 7! ab . We must show that is well-defined. Suppose [a1; b1]; [a2; b2] 2 FD with [a1; b1] = [a2; b2]. Then a1b2 = b1a2. −1 −1 −1 −1 Thus, in E, a1b1 = a2b2 and so (a1b1 ) = (a2b2 ). Now we claim is an injective homomorphism. Let [a; b]; [c; d] 2 FD. Then ([a; b] + [c; d]) = ([ad + bc; bd]) = (ad + bc)(bd)−1 = ab−1 + cd−1 = ([a; b]) + ([c; d]) ([a; b][c; d]) = ([ac; bd]) = (ac)(bd)−1 = (ab−1)(cd−1) = ([a; b]) ([c; d]): For injectivity, suppose ([a; b]) = 0. Then ab−1 = 0. Multiplying both sides by b gives a = 0. Thus, [a; b] = [0; 1], the additive identity in FD, so is injective. Moreover, −1 (φ(a)) = ([a; 1]) = a1 = a: : The previous theorem can be visualized using the following commutative diagram where φ and are as in the theorem and ι is the inclusion map: ι D / E φ 9! FD Remark. It is possible to localize in noncommutative rings but there are several technical hurdles. Example. The field of fractions of Q[x], denoted Q(x), is the set of rational expressions p(x)=q(x) for polynomials p(x); q(x) 2 Q[x] with q(x) 6= 0. 3 2. Factorization Definition 2. Let R be a commutative ring with identity and let a; b 2 R. We say a divides b, denoted a j b, if there exists c 2 R such that b = ac. If there exists a unit u 2 R such that b = au, then a and b are said to be associates. Example. (1) The elements 2 and −2 are associates in Z. In fact, since the only units in Z are ±1, then a; b 2 Z are associates if and only if a = ±b. (2) The elements 2 and 1 are associates in Q since 1 = 2 · (1=2). In fact, if p; q 2 Q are nonzero, then p = q · (p=q) and so any two nonzero elements in Q are associates. Definition 3. Let D be an integral domain. A nonzero element p 2 D that is not a unit is irreducible provided that whenever p = ab, either a or b is a unit. Furthermore, p is prime whenever p j ab either p j a or p j b. 2 2 Example. Let R be the subring of Q[x; y] generated by x ; y , and xy. Then each element is irreducible in R, however xy is not prime because xy divides x2y2 but not x2 or y2. Definition 4. An integral domain D is a unique factorization domain (UFD) if any nonzero, nonunit element a 2 D can be written as a = p1 ··· pk for irreducible elements pi 2 D and if a = q1 ··· q` for irreducibles qj 2 D then k = ` and, up to reordering pi and qi are associates for all i. Example. (1) The integers are a UFD by the Fundamental Theorem of Arithmetic. p (2) The subring [i 3] of is an integral domain (exercise) and the only units are ±1 (also an Z C p p p exercise). The element 4 2 [i 3] has two factorizations: 4 = 2 · 2 = (1 − i 3)(1 + i 3). One can p Z p show that 2; 1 ± i 3 are irreducible. Hence Z[i 3] is not a UFD. Lemma 6. Let D be an integral domain and let a; b 2 D. Then (1) a j b if and only if hbi ⊂ hai. (2) a and b are associates if and only if hbi = hai. (3) a is a unit in D if and only if hai = D. Proof. (1) We have a j b if and only if there exists x 2 D such that ax = b if and only if b 2 hai if and only if hbi ⊂ hai. (2) Suppose a and b are associates. Then there exists a unit y 2 D such that b = ay, thus a j b and so hbi ⊂ hai.
Recommended publications
  • Introduction to Linear Bialgebra
    View metadata, citation and similar papers at core.ac.uk brought to you by CORE provided by University of New Mexico University of New Mexico UNM Digital Repository Mathematics and Statistics Faculty and Staff Publications Academic Department Resources 2005 INTRODUCTION TO LINEAR BIALGEBRA Florentin Smarandache University of New Mexico, [email protected] W.B. Vasantha Kandasamy K. Ilanthenral Follow this and additional works at: https://digitalrepository.unm.edu/math_fsp Part of the Algebra Commons, Analysis Commons, Discrete Mathematics and Combinatorics Commons, and the Other Mathematics Commons Recommended Citation Smarandache, Florentin; W.B. Vasantha Kandasamy; and K. Ilanthenral. "INTRODUCTION TO LINEAR BIALGEBRA." (2005). https://digitalrepository.unm.edu/math_fsp/232 This Book is brought to you for free and open access by the Academic Department Resources at UNM Digital Repository. It has been accepted for inclusion in Mathematics and Statistics Faculty and Staff Publications by an authorized administrator of UNM Digital Repository. For more information, please contact [email protected], [email protected], [email protected]. INTRODUCTION TO LINEAR BIALGEBRA W. B. Vasantha Kandasamy Department of Mathematics Indian Institute of Technology, Madras Chennai – 600036, India e-mail: [email protected] web: http://mat.iitm.ac.in/~wbv Florentin Smarandache Department of Mathematics University of New Mexico Gallup, NM 87301, USA e-mail: [email protected] K. Ilanthenral Editor, Maths Tiger, Quarterly Journal Flat No.11, Mayura Park, 16, Kazhikundram Main Road, Tharamani, Chennai – 600 113, India e-mail: [email protected] HEXIS Phoenix, Arizona 2005 1 This book can be ordered in a paper bound reprint from: Books on Demand ProQuest Information & Learning (University of Microfilm International) 300 N.
    [Show full text]
  • On Free Quasigroups and Quasigroup Representations Stefanie Grace Wang Iowa State University
    Iowa State University Capstones, Theses and Graduate Theses and Dissertations Dissertations 2017 On free quasigroups and quasigroup representations Stefanie Grace Wang Iowa State University Follow this and additional works at: https://lib.dr.iastate.edu/etd Part of the Mathematics Commons Recommended Citation Wang, Stefanie Grace, "On free quasigroups and quasigroup representations" (2017). Graduate Theses and Dissertations. 16298. https://lib.dr.iastate.edu/etd/16298 This Dissertation is brought to you for free and open access by the Iowa State University Capstones, Theses and Dissertations at Iowa State University Digital Repository. It has been accepted for inclusion in Graduate Theses and Dissertations by an authorized administrator of Iowa State University Digital Repository. For more information, please contact [email protected]. On free quasigroups and quasigroup representations by Stefanie Grace Wang A dissertation submitted to the graduate faculty in partial fulfillment of the requirements for the degree of DOCTOR OF PHILOSOPHY Major: Mathematics Program of Study Committee: Jonathan D.H. Smith, Major Professor Jonas Hartwig Justin Peters Yiu Tung Poon Paul Sacks The student author and the program of study committee are solely responsible for the content of this dissertation. The Graduate College will ensure this dissertation is globally accessible and will not permit alterations after a degree is conferred. Iowa State University Ames, Iowa 2017 Copyright c Stefanie Grace Wang, 2017. All rights reserved. ii DEDICATION I would like to dedicate this dissertation to the Integral Liberal Arts Program. The Program changed my life, and I am forever grateful. It is as Aristotle said, \All men by nature desire to know." And Montaigne was certainly correct as well when he said, \There is a plague on Man: his opinion that he knows something." iii TABLE OF CONTENTS LIST OF TABLES .
    [Show full text]
  • Arxiv:2011.04704V2 [Cs.LO] 22 Mar 2021 Eain,Bttre Te Opttoal Neetn Oessuc Models Interesting Well
    Domain Semirings United Uli Fahrenberg1, Christian Johansen2, Georg Struth3, and Krzysztof Ziemia´nski4 1Ecole´ Polytechnique, Palaiseau, France 2 University of Oslo, Norway 3University of Sheffield, UK 4University of Warsaw, Poland Abstract Domain operations on semirings have been axiomatised in two different ways: by a map from an additively idempotent semiring into a boolean subalgebra of the semiring bounded by the additive and multiplicative unit of the semiring, or by an endofunction on a semiring that induces a distributive lattice bounded by the two units as its image. This note presents classes of semirings where these approaches coincide. Keywords: semirings, quantales, domain operations 1 Introduction Domain semirings and Kleene algebras with domain [DMS06, DS11] yield particularly simple program ver- ification formalisms in the style of dynamic logics, algebras of predicate transformers or boolean algebras with operators (which are all related). There are two kinds of axiomatisation. Both are inspired by properties of the domain operation on binary relations, but target other computationally interesting models such as program traces or paths on digraphs as well. The initial two-sorted axiomatisation [DMS06] models the domain operation as a map d : S → B from an additively idempotent semiring (S, +, ·, 0, 1) into a boolean subalgebra B of S bounded by 0 and 1. This seems natural as domain elements form powerset algebras in the target models mentioned. Yet the domain algebra B cannot be chosen freely: B must be the maximal boolean subalgebra of S bounded by 0 and 1 and equal to the set Sd of fixpoints of d in S. The alternative, one-sorted axiomatisation [DS11] therefore models d as an endofunction on a semiring S that induces a suitable domain algebra on Sd—yet generally only a bounded distributive lattice.
    [Show full text]
  • Algebraic Number Theory
    Algebraic Number Theory William B. Hart Warwick Mathematics Institute Abstract. We give a short introduction to algebraic number theory. Algebraic number theory is the study of extension fields Q(α1; α2; : : : ; αn) of the rational numbers, known as algebraic number fields (sometimes number fields for short), in which each of the adjoined complex numbers αi is algebraic, i.e. the root of a polynomial with rational coefficients. Throughout this set of notes we use the notation Z[α1; α2; : : : ; αn] to denote the ring generated by the values αi. It is the smallest ring containing the integers Z and each of the αi. It can be described as the ring of all polynomial expressions in the αi with integer coefficients, i.e. the ring of all expressions built up from elements of Z and the complex numbers αi by finitely many applications of the arithmetic operations of addition and multiplication. The notation Q(α1; α2; : : : ; αn) denotes the field of all quotients of elements of Z[α1; α2; : : : ; αn] with nonzero denominator, i.e. the field of rational functions in the αi, with rational coefficients. It is the smallest field containing the rational numbers Q and all of the αi. It can be thought of as the field of all expressions built up from elements of Z and the numbers αi by finitely many applications of the arithmetic operations of addition, multiplication and division (excepting of course, divide by zero). 1 Algebraic numbers and integers A number α 2 C is called algebraic if it is the root of a monic polynomial n n−1 n−2 f(x) = x + an−1x + an−2x + ::: + a1x + a0 = 0 with rational coefficients ai.
    [Show full text]
  • Fields Besides the Real Numbers Math 130 Linear Algebra
    manner, which are both commutative and asso- ciative, both have identity elements (the additive identity denoted 0 and the multiplicative identity denoted 1), addition has inverse elements (the ad- ditive inverse of x denoted −x as usual), multipli- cation has inverses of nonzero elements (the multi- Fields besides the Real Numbers 1 −1 plicative inverse of x denoted x or x ), multipli- Math 130 Linear Algebra cation distributes over addition, and 0 6= 1. D Joyce, Fall 2015 Of course, one example of a field is the field of Most of the time in linear algebra, our vectors real numbers R. What are some others? will have coordinates that are real numbers, that is to say, our scalar field is R, the real numbers. Example 2 (The field of rational numbers, Q). Another example is the field of rational numbers. But linear algebra works over other fields, too, A rational number is the quotient of two integers like C, the complex numbers. In fact, when we a=b where the denominator is not 0. The set of discuss eigenvalues and eigenvectors, we'll need to all rational numbers is denoted Q. We're familiar do linear algebra over C. Some of the applications with the fact that the sum, difference, product, and of linear algebra such as solving linear differential quotient (when the denominator is not zero) of ra- equations require C as as well. tional numbers is another rational number, so Q Some applications in computer science use linear has all the operations it needs to be a field, and algebra over a two-element field Z (described be- 2 since it's part of the field of the real numbers R, its low).
    [Show full text]
  • Ring (Mathematics) 1 Ring (Mathematics)
    Ring (mathematics) 1 Ring (mathematics) In mathematics, a ring is an algebraic structure consisting of a set together with two binary operations usually called addition and multiplication, where the set is an abelian group under addition (called the additive group of the ring) and a monoid under multiplication such that multiplication distributes over addition.a[›] In other words the ring axioms require that addition is commutative, addition and multiplication are associative, multiplication distributes over addition, each element in the set has an additive inverse, and there exists an additive identity. One of the most common examples of a ring is the set of integers endowed with its natural operations of addition and multiplication. Certain variations of the definition of a ring are sometimes employed, and these are outlined later in the article. Polynomials, represented here by curves, form a ring under addition The branch of mathematics that studies rings is known and multiplication. as ring theory. Ring theorists study properties common to both familiar mathematical structures such as integers and polynomials, and to the many less well-known mathematical structures that also satisfy the axioms of ring theory. The ubiquity of rings makes them a central organizing principle of contemporary mathematics.[1] Ring theory may be used to understand fundamental physical laws, such as those underlying special relativity and symmetry phenomena in molecular chemistry. The concept of a ring first arose from attempts to prove Fermat's last theorem, starting with Richard Dedekind in the 1880s. After contributions from other fields, mainly number theory, the ring notion was generalized and firmly established during the 1920s by Emmy Noether and Wolfgang Krull.[2] Modern ring theory—a very active mathematical discipline—studies rings in their own right.
    [Show full text]
  • A Brief History of Ring Theory
    A Brief History of Ring Theory by Kristen Pollock Abstract Algebra II, Math 442 Loyola College, Spring 2005 A Brief History of Ring Theory Kristen Pollock 2 1. Introduction In order to fully define and examine an abstract ring, this essay will follow a procedure that is unlike a typical algebra textbook. That is, rather than initially offering just definitions, relevant examples will first be supplied so that the origins of a ring and its components can be better understood. Of course, this is the path that history has taken so what better way to proceed? First, it is important to understand that the abstract ring concept emerged from not one, but two theories: commutative ring theory and noncommutative ring the- ory. These two theories originated in different problems, were developed by different people and flourished in different directions. Still, these theories have much in com- mon and together form the foundation of today's ring theory. Specifically, modern commutative ring theory has its roots in problems of algebraic number theory and algebraic geometry. On the other hand, noncommutative ring theory originated from an attempt to expand the complex numbers to a variety of hypercomplex number systems. 2. Noncommutative Rings We will begin with noncommutative ring theory and its main originating ex- ample: the quaternions. According to Israel Kleiner's article \The Genesis of the Abstract Ring Concept," [2]. these numbers, created by Hamilton in 1843, are of the form a + bi + cj + dk (a; b; c; d 2 R) where addition is through its components 2 2 2 and multiplication is subject to the relations i =pj = k = ijk = −1.
    [Show full text]
  • Subrings, Ideals and Quotient Rings the First Definition Should Not Be
    Section 17: Subrings, Ideals and Quotient Rings The first definition should not be unexpected: Def: A nonempty subset S of a ring R is a subring of R if S is closed under addition, negatives (so it's an additive subgroup) and multiplication; in other words, S inherits operations from R that make it a ring in its own right. Naturally, Z is a subring of Q, which is a subring of R, which is a subring of C. Also, R is a subring of R[x], which is a subring of R[x; y], etc. The additive subgroups nZ of Z are subrings of Z | the product of two multiples of n is another multiple of n. For the same reason, the subgroups hdi in the various Zn's are subrings. Most of these latter subrings do not have unities. But we know that, in the ring Z24, 9 is an idempotent, as is 16 = 1 − 9. In the subrings h9i and h16i of Z24, 9 and 16 respectively are unities. The subgroup h1=2i of Q is not a subring of Q because it is not closed under multiplication: (1=2)2 = 1=4 is not an integer multiple of 1=2. Of course the immediate next question is which subrings can be used to form factor rings, as normal subgroups allowed us to form factor groups. Because a ring is commutative as an additive group, normality is not a problem; so we are really asking when does multiplication of additive cosets S + a, done by multiplying their representatives, (S + a)(S + b) = S + (ab), make sense? Again, it's a question of whether this operation is well-defined: If S + a = S + c and S + b = S + d, what must be true about S so that we can be sure S + (ab) = S + (cd)? Using the definition of cosets: If a − c; b − d 2 S, what must be true about S to assure that ab − cd 2 S? We need to have the following element always end up in S: ab − cd = ab − ad + ad − cd = a(b − d) + (a − c)d : Because b − d and a − c can be any elements of S (and either one may be 0), and a; d can be any elements of R, the property required to assure that this element is in S, and hence that this multiplication of cosets is well-defined, is that, for all s in S and r in R, sr and rs are also in S.
    [Show full text]
  • Define the Determinant of A, to Be Det(A) = Ad − Bc. EX
    DETERMINANT 1. 2 × 2 Determinants Fix a matrix A 2 R2×2 a b A = c d Define the determinant of A, to be det(A) = ad − bc: 2 −1 EXAMPLE: det = 2(2) − (−1)(−4) = 0. −4 2 det(A) encodes important geometric and algebraic information about A. For instance, the matrix A is invertible if and only if det(A) 6= 0. To see this suppose det(A) 6= 0, in this case the matrix 1 d −b B = det A −c a is well-defined. One computes, 1 ad − bc 0 BA = = I : ad − bc 0 ad − bc 2 and so A is invertible and A−1 = B. In the other direction, if A is not invertible, then the columns are linearly dependent and so either a = kb and c = kd or b = ka and d = kc for some k 2 R. Hence, det(A) = kbd − kbd = 0 or = kac − kac = 0. More geometrically, if x1 S = : 0 ≤ x1; x2 ≤ 1 x2 is the unit square and A(S) = fA~x : ~x 2 Sg is the image under multiplication by A of S, then the area of A(S), which we denote by jA(S)j is jA(S)j = j det(A)j: 2. Determinants of n × n matrices We seek a good notion for det(A) when A 2 Rn×n. It is improtant to remember that while this is of historical and theoretical importance, it is not as significant for computational purposes. Begin by fixing a matrix A 2 Rn×n of the form 2 3 a11 ··· a1n 6 .
    [Show full text]
  • EXAMPLES of CHAIN DOMAINS 1. Introduction In
    PROCEEDINGS OF THE AMERICAN MATHEMATICAL SOCIETY Volume 126, Number 3, March 1998, Pages 661{667 S 0002-9939(98)04127-6 EXAMPLES OF CHAIN DOMAINS R. MAZUREK AND E. ROSZKOWSKA (Communicated by Ken Goodearl) Abstract. Let γ be a nonzero ordinal such that α + γ = γ for every ordinal α<γ. A chain domain R (i.e. a domain with linearly ordered lattices of left ideals and right ideals) is constructed such that R is isomorphic with all its nonzero factor-rings and γ is the ordinal type of the set of proper ideals of R. The construction provides answers to some open questions. 1. Introduction In [6] Leavitt and van Leeuwen studied the class of rings which are isomorphic with all nonzero factor-rings. They proved that forK every ring R the set of ideals of R is well-ordered and represented by a prime component∈K ordinal γ (i.e. γ>0andα+γ=γfor every ordinal α<γ). In this paper we show that the class contains remarkable examples of rings. Namely, for every prime component ordinalK γ we construct a chain domain R (i.e. a domain whose lattice of left ideals as well as the lattice of right ideals are linearly ordered) such that R and γ is the ordinal type of the set of proper ideals of R. We begin the construction∈K by selecting a semigroup that has properties analogous to those we want R to possess ( 2). The desired ring R is the Jacobson radical of a localization of a semigroup ring§ of the selected semigroup with respect to an Ore set ( 3).
    [Show full text]
  • Number Fields
    Part II | Number Fields Based on lectures by I. Grojnowski Notes taken by Dexter Chua Lent 2016 These notes are not endorsed by the lecturers, and I have modified them (often significantly) after lectures. They are nowhere near accurate representations of what was actually lectured, and in particular, all errors are almost surely mine. Part IB Groups, Rings and Modules is essential and Part II Galois Theory is desirable Definition of algebraic number fields, their integers and units. Norms, bases and discriminants. [3] Ideals, principal and prime ideals, unique factorisation. Norms of ideals. [3] Minkowski's theorem on convex bodies. Statement of Dirichlet's unit theorem. Deter- mination of units in quadratic fields. [2] Ideal classes, finiteness of the class group. Calculation of class numbers using statement of the Minkowski bound. [3] Dedekind's theorem on the factorisation of primes. Application to quadratic fields. [2] Discussion of the cyclotomic field and the Fermat equation or some other topic chosen by the lecturer. [3] 1 Contents II Number Fields Contents 0 Introduction 3 1 Number fields 4 2 Norm, trace, discriminant, numbers 10 3 Multiplicative structure of ideals 17 4 Norms of ideals 27 5 Structure of prime ideals 32 6 Minkowski bound and finiteness of class group 37 7 Dirichlet's unit theorem 48 8 L-functions, Dirichlet series* 56 Index 68 2 0 Introduction II Number Fields 0 Introduction Technically, IID Galois Theory is not a prerequisite of this course. However, many results we have are analogous to what we did in Galois Theory, and we will not refrain from pointing out the correspondence.
    [Show full text]
  • Free Medial Quandles
    Algebra Univers. 78 (2017) 43–54 DOI 10.1007/s00012-017-0443-2 Published online May 23, 2017 © 2017 The Author(s) Algebra Universalis This article is an open access publication Free medial quandles Premyslˇ Jedlicka,ˇ Agata Pilitowska, and Anna Zamojska-Dzienio Abstract. This paper gives the construction of free medial quandles as well as free n-symmetric medial quandles and free m-reductive medial quandles. 1. Introduction A binary algebra (Q, ) is called a rack if the following conditions hold, for · every x, y, z Q: ∈ x(yz)=(xy)(xz) (we say Q is left distributive), • the equation xu = y has a unique solution u Q (we say Q is a left • ∈ quasigroup). An idempotent rack is called a quandle (we say Q is idempotent if xx = x for every x Q). A quandle Q is medial if, for every x, y, u, v Q, ∈ ∈ (xy)(uv)=(xu)(yv). An important example of a medial quandle is an abelian group A with an operation defined by a b = (1 h)(a)+h(b), where h is an automorphism ∗ ∗ − of A. This construction is called an affine quandle (or sometimes an Alexander quandle) and denoted by Aff(A, h). In the literature [6, 7], the group A is 1 usually considered to be a Z[t, t− ]-module, where t a = h(a), for each a A. · ∈ We shall adopt this point of view here as well and we usually write Aff(A, r) instead, where r is a ring element. Note that in universal algebra terminology, an algebra is said to be affine if it is polynomially equivalent to a module.
    [Show full text]