Chapter 2 Rings and Modules

Total Page:16

File Type:pdf, Size:1020Kb

Chapter 2 Rings and Modules Chapter 2 Rings and Modules 2.1 Rings Definition 2.1.1. A ring consists of a set R together with binary operations + and · satisfying: 1. (R; +) forms an abelian group, 2. (a · b) · c = a · (b · c) 8a; b; c 2 R, 3. 91 =6 0 2 R such that a · 1 = 1 · a = a 8a 2 R, and 4. a · (b + c) = a · b + a · c and (a + b) · c = a · c + b · c 8a; b; c 2 R. Note: 1. Some people (e.g. Dummit + Foote) do not require condition 3, and refer to a \ring with identity" if they want to assume · has an identity element. 2. People who include existence of a unit in their defn. of a ring refer to a \ring without identity" for an object satisfying the other three axioms. Some people (e.g. Jacobson) call this a \rng". 3. Some people (e.g. Lang) do not require 1 =6 0 in condition 3. Definition 2.1.2. R is called commutative if its multiplication is commutative, ie. ab = ba 8a; b 2 R: Definition 2.1.3. A ring homomorphism from R to S is a function f : R 7! S such that 8a; b 2 R: 55 1. f(a + b) = f(a) + f(b), 2. f(ab) = f(a)f(b), and 3. f(1) = 1. A bijective ring homomorphism is called an isomorphism. Definition 2.1.4. A subring of R is a subset A which forms a ring such that the inclusion A ,! R is a ring homomorphism. A subgroup I of the abelian group (R; +) is called a (two - sided) ideal if x 2 I; r 2 R ) rx 2 I and xr 2 I: Similarly if a subgroup I satisfies x 2 I; r 2 R ) rx 2 I; I is called a left ideal, and if it satisfies x 2 I; r 2 R ) xr 2 I; it is called a right ideal. Example 2.1.5. If f : R 7! S is a homomorphism then ker f := fx 2 R j f(x) = 0g is an ideal in R. (An ideal is always a subrng but never a subring, unless it is all of R.) Theorem 2.1.6. Let I⊆R be a proper ideal. Then 9 a ring R=I and a surjective ring homo- morphism f : R 7!! R=I such that ker f = I. Proof. Define an equivalence relation on R by x ∼ y () x − y 2 I. Let R=I := fequiv. classesg: Define operations on R=I by [x] + [y] := [x + y]; [x] · [y] := [xy]: Check that these are well-defined and produce a ring structure on R=I. Define f : R 7! R=I by f(x) = [x]. f is a ring homomorphism. Moreover, f(x) = 0 iff [x] = 0 iff x = x − 0 2 I. 56 Definition 2.1.7. The ring R is called a division ring if (R − f0g; ·) forms a group. A commutative division ring is called a field. An element u 2 R for which 9v 2 R such that uv = vu = 1 is called a unit. Notation: R× = funits of Rg: This forms a group under multiplication. A non-zero element x 2 R is called a zero divisor if 9y =6 0 such that either xy = 0 or yx = 0. A commutative ring with no zero divisors is called an integral domain. Proposition 2.1.8. If x =6 0 is not a zero divisor and xy = xz then y = z. Proof. x(y − z) = 0 and x is not a zero divisor so either x = 0 or y − z = 0. But x =6 0 so y = z. Theorem 2.1.9 (First Isomorphism Theorem). Let f : R 7! S be a ring homomorphism. Then R= ker f =∼ Imf. Theorem 2.1.10 (Second Isomorphism Theorem). Let A ⊂ R be a subring and let I⊆R be a proper ideal. Then A + I := fa + x j a 2 A; x 2 Ig is a subring of R, A \ I is a proper ideal in A, and (A + I)=I ∼= A=(A \ I): Theorem 2.1.11 (Third Isomorphism Theorem). Let I ⊂ J be proper ideals of R. Then J=I := f[x] 2 R=I j x 2 Jg is an ideal in R=I, and R=I ∼= R=J: J=I Theorem 2.1.12 (Fourth Isomorphism Theorem). Let I be a proper ideal of R. Then the correspondence J 7! J=I is a bijection between the ideals of J containing I and the ideals of R=I. Let I; J be ideals in R. Define ideals I + J := fx + y j x 2 I; y 2 Jg; I \ J; n IJ := xiyy j n 2 N; xi 2 I; yi 2 J ( i=1 ) X Then IJ ⊂ I \ J ⊂ I [ J ⊂ I + J: (Note that I [ J may not be an ideal.) I + J is the smallest ideal containing both I and J. 57 2.2 Maximal and Prime Ideals Definition 2.2.1. An ideal M⊆R is called a maximal ideal if @ an ideal I s.t. M⊆I⊆R. Lemma 2.2.2. Given an ideal I⊆R, 9 a maximal ideal M s.t. I ⊂ M. Proof. Let S = fideals J j I ⊂ J⊆Rg: Then S is a partially ordered set (ordered by inclusion). If C ⊂ S is a chain (ie. a totally ordered subset) then J = C C [2C is an ideal which forms an upper bound for C in S (it is indeed a proper ideal since 1 62 J). ) Zorn's Lemma ) S has a maximal element M. For the rest of this section, suppose that R is commutative. Proposition 2.2.3. R is a field () the only ideals of R are f0g and R. Proof. ): Let R be a field and let I ⊂ R be an ideal. If I =6 f0g then 9x =6 0 2 I. R a field ) 9y 2 R such that xy = yx = 1. Since I is an ideal, 1 2 I, so r 2 I 8r 2 R. Thus I = R. (: Suppose the only ideals in R are f0g and R. Let x =6 0 2 R. Let I = Rx := frx j r 2 Rg: I is an ideal and x = 1x 2 R, so I =6 0. Hence I = R, so 1 2 I. ie. 1 = yz for some y 2 R. ) Every x =6 0 2 R has an inverse, so R is a field. Corollary 2.2.4. Let f : F 7! S be a ring homomorphism where F is a field. Then f is injective. Proof. ker f is a proper ideal in F , so ker f = 0. Theorem 2.2.5. M is a maximal ideal () R=M is a field. 58 Proof. The 4th iso. thm. says 9 a bijection between the ideals of R containing M and the ideals of R=M. ) 9I s.t. M⊆I⊆R () 9J s.t. f0}⊆J⊆R=M. ie. M is not maximal () R=M is not a field. Definition 2.2.6. An ideal P⊆R is called a prime ideal if ab 2 P implies a 2 P or b 2 P. Theorem 2.2.7. P is a prime ideal () R=P is an integral domain. Proof. ): Suppose P is a prime ideal. If [xy] = [x][y] = 0 in R=P then xy 2 P, so either x 2 P or y 2 P. ie. either [x] = 0 or [y] = 0. Thus R=P has no zero divisors. (: Suppose R=P is an integral domain. If xy 2 P then [x][y] = 0 in R=P, so [x] = 0 or [y] = 0. ie. either x 2 P or y 2 P. Corollary 2.2.8. A maximal ideal is a prime ideal. Proof. A field is an integral domain. Notation: a j b means 9c s.t. b = ac (say a divides b). Proposition 2.2.9. In an integral domain, if a j b and b j a then b = ua for some unit u. Proof. a j b ) b = ua for some u 2 R. b j a ) a = vb for some v 2 R. ) b = ua = uvb, and since b is not a zero divisor, 1 = uv. Thus, u is a unit. Definition 2.2.10. q is called a greatest common divisor of a and b if: 1. q j a and q j b, and 2. If c also satisfies c j a; c j b then c j q. Notation: q = (a; b) means q is the greatest common divisor of a and b. We say a and b are relatively prime if (a; b) = 1. Proposition 2.2.11. Let R be an integral domain. If q = (a; b) and q0 = (a; b) then q0 = uq for some unit u. Conversely, if q = (a; b) and q0 = uq where u is a unit then q0 = (a; b). Proof. Let q = (a; b). If q0 = (a; b) then q0 j q and q j q0 so q0 = uq for some unit u. Conversely, if q0 = uq for some unit u then q0 j q so q0 j a and q0 j b. Also q j q0 so whenever c j a and c j b, c j q so c j q0. 59 Definition 2.2.12. A non-unit p =6 0 2 R is called a prime if p j ab ) p j a or p j b.
Recommended publications
  • Modules and Vector Spaces
    Modules and Vector Spaces R. C. Daileda October 16, 2017 1 Modules Definition 1. A (left) R-module is a triple (R; M; ·) consisting of a ring R, an (additive) abelian group M and a binary operation · : R × M ! M (simply written as r · m = rm) that for all r; s 2 R and m; n 2 M satisfies • r(m + n) = rm + rn ; • (r + s)m = rm + sm ; • r(sm) = (rs)m. If R has unity we also require that 1m = m for all m 2 M. If R = F , a field, we call M a vector space (over F ). N Remark 1. One can show that as a consequence of this definition, the zeros of R and M both \act like zero" relative to the binary operation between R and M, i.e. 0Rm = 0M and r0M = 0M for all r 2 R and m 2 M. H Example 1. Let R be a ring. • R is an R-module using multiplication in R as the binary operation. • Every (additive) abelian group G is a Z-module via n · g = ng for n 2 Z and g 2 G. In fact, this is the only way to make G into a Z-module. Since we must have 1 · g = g for all g 2 G, one can show that n · g = ng for all n 2 Z. Thus there is only one possible Z-module structure on any abelian group. • Rn = R ⊕ R ⊕ · · · ⊕ R is an R-module via | {z } n times r(a1; a2; : : : ; an) = (ra1; ra2; : : : ; ran): • Mn(R) is an R-module via r(aij) = (raij): • R[x] is an R-module via X i X i r aix = raix : i i • Every ideal in R is an R-module.
    [Show full text]
  • 6. Localization
    52 Andreas Gathmann 6. Localization Localization is a very powerful technique in commutative algebra that often allows to reduce ques- tions on rings and modules to a union of smaller “local” problems. It can easily be motivated both from an algebraic and a geometric point of view, so let us start by explaining the idea behind it in these two settings. Remark 6.1 (Motivation for localization). (a) Algebraic motivation: Let R be a ring which is not a field, i. e. in which not all non-zero elements are units. The algebraic idea of localization is then to make more (or even all) non-zero elements invertible by introducing fractions, in the same way as one passes from the integers Z to the rational numbers Q. Let us have a more precise look at this particular example: in order to construct the rational numbers from the integers we start with R = Z, and let S = Znf0g be the subset of the elements of R that we would like to become invertible. On the set R×S we then consider the equivalence relation (a;s) ∼ (a0;s0) , as0 − a0s = 0 a and denote the equivalence class of a pair (a;s) by s . The set of these “fractions” is then obviously Q, and we can define addition and multiplication on it in the expected way by a a0 as0+a0s a a0 aa0 s + s0 := ss0 and s · s0 := ss0 . (b) Geometric motivation: Now let R = A(X) be the ring of polynomial functions on a variety X. In the same way as in (a) we can ask if it makes sense to consider fractions of such polynomials, i.
    [Show full text]
  • 11. Finitely-Generated Modules
    11. Finitely-generated modules 11.1 Free modules 11.2 Finitely-generated modules over domains 11.3 PIDs are UFDs 11.4 Structure theorem, again 11.5 Recovering the earlier structure theorem 11.6 Submodules of free modules 1. Free modules The following definition is an example of defining things by mapping properties, that is, by the way the object relates to other objects, rather than by internal structure. The first proposition, which says that there is at most one such thing, is typical, as is its proof. Let R be a commutative ring with 1. Let S be a set. A free R-module M on generators S is an R-module M and a set map i : S −! M such that, for any R-module N and any set map f : S −! N, there is a unique R-module homomorphism f~ : M −! N such that f~◦ i = f : S −! N The elements of i(S) in M are an R-basis for M. [1.0.1] Proposition: If a free R-module M on generators S exists, it is unique up to unique isomorphism. Proof: First, we claim that the only R-module homomorphism F : M −! M such that F ◦ i = i is the identity map. Indeed, by definition, [1] given i : S −! M there is a unique ~i : M −! M such that ~i ◦ i = i. The identity map on M certainly meets this requirement, so, by uniqueness, ~i can only be the identity. Now let M 0 be another free module on generators S, with i0 : S −! M 0 as in the definition.
    [Show full text]
  • Commutative Algebra
    Commutative Algebra Andrew Kobin Spring 2016 / 2019 Contents Contents Contents 1 Preliminaries 1 1.1 Radicals . .1 1.2 Nakayama's Lemma and Consequences . .4 1.3 Localization . .5 1.4 Transcendence Degree . 10 2 Integral Dependence 14 2.1 Integral Extensions of Rings . 14 2.2 Integrality and Field Extensions . 18 2.3 Integrality, Ideals and Localization . 21 2.4 Normalization . 28 2.5 Valuation Rings . 32 2.6 Dimension and Transcendence Degree . 33 3 Noetherian and Artinian Rings 37 3.1 Ascending and Descending Chains . 37 3.2 Composition Series . 40 3.3 Noetherian Rings . 42 3.4 Primary Decomposition . 46 3.5 Artinian Rings . 53 3.6 Associated Primes . 56 4 Discrete Valuations and Dedekind Domains 60 4.1 Discrete Valuation Rings . 60 4.2 Dedekind Domains . 64 4.3 Fractional and Invertible Ideals . 65 4.4 The Class Group . 70 4.5 Dedekind Domains in Extensions . 72 5 Completion and Filtration 76 5.1 Topological Abelian Groups and Completion . 76 5.2 Inverse Limits . 78 5.3 Topological Rings and Module Filtrations . 82 5.4 Graded Rings and Modules . 84 6 Dimension Theory 89 6.1 Hilbert Functions . 89 6.2 Local Noetherian Rings . 94 6.3 Complete Local Rings . 98 7 Singularities 106 7.1 Derived Functors . 106 7.2 Regular Sequences and the Koszul Complex . 109 7.3 Projective Dimension . 114 i Contents Contents 7.4 Depth and Cohen-Macauley Rings . 118 7.5 Gorenstein Rings . 127 8 Algebraic Geometry 133 8.1 Affine Algebraic Varieties . 133 8.2 Morphisms of Affine Varieties . 142 8.3 Sheaves of Functions .
    [Show full text]
  • NOTES in COMMUTATIVE ALGEBRA: PART 1 1. Results/Definitions Of
    NOTES IN COMMUTATIVE ALGEBRA: PART 1 KELLER VANDEBOGERT 1. Results/Definitions of Ring Theory It is in this section that a collection of standard results and definitions in commutative ring theory will be presented. For the rest of this paper, any ring R will be assumed commutative with identity. We shall also use "=" and "∼=" (isomorphism) interchangeably, where the context should make the meaning clear. 1.1. The Basics. Definition 1.1. A maximal ideal is any proper ideal that is not con- tained in any strictly larger proper ideal. The set of maximal ideals of a ring R is denoted m-Spec(R). Definition 1.2. A prime ideal p is such that for any a, b 2 R, ab 2 p implies that a or b 2 p. The set of prime ideals of R is denoted Spec(R). p Definition 1.3. The radical of an ideal I, denoted I, is the set of a 2 R such that an 2 I for some positive integer n. Definition 1.4. A primary ideal p is an ideal such that if ab 2 p and a2 = p, then bn 2 p for some positive integer n. In particular, any maximal ideal is prime, and the radical of a pri- mary ideal is prime. Date: September 3, 2017. 1 2 KELLER VANDEBOGERT Definition 1.5. The notation (R; m; k) shall denote the local ring R which has unique maximal ideal m and residue field k := R=m. Example 1.6. Consider the set of smooth functions on a manifold M.
    [Show full text]
  • MATH 210A, FALL 2017 Question 1. Consider a Short Exact Sequence 0
    MATH 210A, FALL 2017 HW 3 SOLUTIONS WRITTEN BY DAN DORE, EDITS BY PROF.CHURCH (If you find any errors, please email [email protected]) α β Question 1. Consider a short exact sequence 0 ! A −! B −! C ! 0. Prove that the following are equivalent. (A) There exists a homomorphism σ : C ! B such that β ◦ σ = idC . (B) There exists a homomorphism τ : B ! A such that τ ◦ α = idA. (C) There exists an isomorphism ': B ! A ⊕ C under which α corresponds to the inclusion A,! A ⊕ C and β corresponds to the projection A ⊕ C C. α β When these equivalent conditions hold, we say the short exact sequence 0 ! A −! B −! C ! 0 splits. We can also equivalently say “β : B ! C splits” (since by (i) this only depends on β) or “α: A ! B splits” (by (ii)). Solution. (A) =) (B): Let σ : C ! B be such that β ◦ σ = idC . Then we can define a homomorphism P : B ! B by P = idB −σ ◦ β. We should think of this as a projection onto A, in that P maps B into the submodule A and it is the identity on A (which is exactly what we’re trying to prove). Equivalently, we must show P ◦ P = P and im(P ) = A. It’s often useful to recognize the fact that a submodule A ⊆ B is a direct summand iff there is such a projection. Now, let’s prove that P is a projection. We have β ◦ P = β − β ◦ σ ◦ β = β − idC ◦β = 0. Thus, by the universal property of the kernel (as developed in HW2), P factors through the kernel α: A ! B.
    [Show full text]
  • On Quotient Modules – the Case of Arbitrary Multiplicity
    On quotient modules – the case of arbitrary multiplicity Ronald G. Douglas∗ Texas A & M University College Station Texas 77843 Gadadhar Misra†and Cherian Varughese Indian Statistical Institute R. V. College Post Bangalore 560 059 Abstract: Let M be a Hilbert module of holomorphic functions defined m on a bounded domain Ω ⊆ C . Let M0 be the submodule of functions vanishing to order k on a hypersurface Z in Ω. In this paper, we describe the quotient module Mq. Introduction If M is a Hilbert module over a function algebra A and M0 ⊆ M is a submodule, then determining the quotient module Mq is an interesting problem, particularly if the function algebra consists of holomorphic functions on a domain Ω in Cm and M is a functional Hilbert space. It would be very desirable to describe the quotient module Mq in terms of the last two terms in the short exact sequence X 0 ←− Mq ←− M ←− M0 ←− 0 where X is the inclusion map. For certain modules over the disc algebra, this is related to the model theory of Sz.-Nagy and Foias. In a previous paper [6], the quotient module was described assuming that the sub- module M0 is the maximal set of functions in M vanishing on Z, where Z is an analytic ∗The research for this paper was partly carried out during a visit to ISI - Bangalore in January 1996 with financial support from the Indian Statistical Institute and the International Mathematical Union. †The research for this paper was partly carried out during a visit to Texas A&M University in August, 1997 with financial support from Texas A&M University.
    [Show full text]
  • On the Derived Quotient Moduleo
    transactions of the american mathematical society Volume 154, February 1971 ON THE DERIVED QUOTIENT MODULEO BY C. N. WINTON Abstract. With every Ä-module M associate the direct limit of Horn« (D, M) over the dense right ideals of R, the derived quotient module SHiM) of M. 3>(M) is a module over the complete ring of right quotients of R. Relationships between Si(M) and the torsion theory of Gentile-Jans are explored and functorial properties of S> are discussed. When M is torsion free, results are given concerning rational closure, rational completion, and injectivity. 1. Introduction. Let R be a ring with unity and let Q be its complete ring of right quotients. Following Lambek [8], a right ideal D of R is called dense provided that if an R-map f: E(RB) ->■E(RR), where E(RR) denotes the injective hull of RR, is such thatfi(D) = 0, then/=0. It is easy to see this is equivalent to xZ)^(O) for every xe E(RB). The collection of dense right ideals is closed under finite intersection; furthermore, any right ideal containing a dense right ideal is again dense. Hence, the collection becomes a directed set if we let Dy á D2 whenever D2 £ Dy for dense right ideals Dy and D2 of R. It follows that for any /{-module M we can form the direct limit £>(M) of {HomB (D, M) \ D is a dense right ideal of R} over the directed set of dense right ideals of R. We will call 3>(M) the derived quotient module of M.
    [Show full text]
  • Part IB — Groups, Rings and Modules
    Part IB | Groups, Rings and Modules Based on lectures by O. Randal-Williams 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. Groups Basic concepts of group theory recalled from Part IA Groups. Normal subgroups, quotient groups and isomorphism theorems. Permutation groups. Groups acting on sets, permutation representations. Conjugacy classes, centralizers and normalizers. The centre of a group. Elementary properties of finite p-groups. Examples of finite linear groups and groups arising from geometry. Simplicity of An. Sylow subgroups and Sylow theorems. Applications, groups of small order. [8] Rings Definition and examples of rings (commutative, with 1). Ideals, homomorphisms, quotient rings, isomorphism theorems. Prime and maximal ideals. Fields. The characteristic of a field. Field of fractions of an integral domain. Factorization in rings; units, primes and irreducibles. Unique factorization in principal ideal domains, and in polynomial rings. Gauss' Lemma and Eisenstein's irreducibility criterion. Rings Z[α] of algebraic integers as subsets of C and quotients of Z[x]. Examples of Euclidean domains and uniqueness and non-uniqueness of factorization. Factorization in the ring of Gaussian integers; representation of integers as sums of two squares. Ideals in polynomial rings. Hilbert basis theorem. [10] Modules Definitions, examples of vector spaces, abelian groups and vector spaces with an endomorphism. Sub-modules, homomorphisms, quotient modules and direct sums. Equivalence of matrices, canonical form. Structure of finitely generated modules over Euclidean domains, applications to abelian groups and Jordan normal form.
    [Show full text]
  • Ring and Module Theory Qual Review
    Ring and Module Theory Qual Review Robert Won Prof. Rogalski 1 (Some) qual problems (Spring 2007, 2) Let I;J be two ideals in a commutative ring R (with unit). (a) Define K = fr : rJ ≤ Ig. Show that K is an ideal (b) If R is a PID, so I = hii, J = hji, give a formula for a generator k of K. (Spring 2007, 3) Describe up to isomorphism all the R[x]-module structures one might put on a 3 dimensional real vector space (extending the R action). Fundamental theorem of modules over a PID. Choose your favorite canonical form. Note that R[x] is infinite dimensional so an R[x]-module must be a direct sum of R[x]=(ai) (which has dimension deg ai). The dimensions must sum to three. (Fall 2009, 8) Let R be a commutative ring with identity. Suppose I and J are ideals of R such that R=I and R=J are noetherian rings. Prove that R=(I \ J) is also a noetherian ring. (Spring 2012, 3) Let R be a commutative ring. (a) Suppose that R is noetherian. Show that if ' : R ! R is a surjective ring homomor- phism, then it is injective. Construct an ascending chain by taking nested kernels. Use ACC. (b) If R is not noetherian, must a surjective ring homomorphism be injective? Prove or give a counterexample. Noetherianness is some finiteness condition, so it stands to reason that part (a) is true. Part (b) can't possibly be, because rings can be big. You should know an example of a non-noetherian commutative ring, F [x1; x2;::: ], the polynomial ring in countably many variables.
    [Show full text]
  • Linear Source Invertible Bimodules and Green Correspondence
    Linear source invertible bimodules and Green correspondence Markus Linckelmann and Michael Livesey April 22, 2020 Abstract We show that the Green correspondence induces an injective group homomorphism from the linear source Picard group L(B) of a block B of a finite group algebra to the linear source Picard group L(C), where C is the Brauer correspondent of B. This homomorphism maps the trivial source Picard group T (B) to the trivial source Picard group T (C). We show further that the endopermutation source Picard group E(B) is bounded in terms of the defect groups of B and that when B has a normal defect group E(B) = L(B). Finally we prove that the rank of any invertible B-bimodule is bounded by that of B. 1 Introduction Let p be a prime and k a perfect field of characteristic p. We denote by O either a complete discrete valuation ring with maximal ideal J(O) = πO for some π ∈ O, with residue field k and field of fractions K of characteristic zero, or O = k. We make the blanket assumption that k and K are large enough for the finite groups and their subgroups in the statements below. Let A be an O-algebra. An A-A-bimodule M is called invertible if M is finitely generated projective as a left A-module, as a right A-module, and if there exits an A-A-bimodule N which is finitely generated projective as a left and right A-module such that M ⊗A N =∼ A =∼ N ⊗A M as A-A-bimodules.
    [Show full text]
  • Module Theory
    Module Theory Claudia Menini 2014-2015 Contents Contents 2 1 Modules 4 1.1 Homomorphisms and Quotients ..................... 4 1.2 Quotient Module and Isomorphism Theorems . 10 1.3 Product and Direct Sum of a Family of Modules . 13 1.4 Sum and Direct Sum of Submodules. Cyclic Modules . 21 1.5 Exact sequences and split exact sequences . 27 1.6 HomR (M; N) ............................... 32 2 Free and projective modules 35 3 Injective Modules and Injective Envelopes 41 4 Generators and Cogenerators 59 5 2 × 2 Matrix Ring 65 6 Tensor Product and bimodules 68 6.1 Tensor Product 1 ............................. 68 6.2 Bimodules ................................. 78 6.3 Tensor Product 2 ............................. 82 7 Homology 94 7.1 Categories and Functors ......................... 94 7.2 Snake Lemma ...............................100 7.3 Chain Complexes .............................105 7.4 Homotopies ................................113 7.5 Projective resolutions . 116 7.6 Left Derived functors . 123 7.7 Cochain Complexes and Right Derived Functors . 139 8 Semisimple modules and Jacobson radical 145 9 Chain Conditions. 160 2 CONTENTS 3 10 Progenerators and Morita Equivalence 173 10.1 Progenerators ...............................173 10.2 Frobenius .................................199 Chapter 1 Modules 1.1 Homomorphisms and Quotients R Definition 1.1. Let R be a ring. A left R-module is a pair (M; µM ) where (M+; 0) is an abelian group and R µ = µM : R × M ! M is a map such that, setting a · x = µ ((a; x)) , the following properties are satisfied : M1 a · (x + y) = a · x + a · y; M2 (a + b) · x = a · x + b · x; M3 (a ·R b) x = a · (b · x); M4 1R · x = x for every a; b 2 R and every x; y 2 M.
    [Show full text]