Abstract Algebra/Modules

From testwiki
Revision as of 09:01, 14 August 2022 by imported>SHB2000 (obervant->observant - Fix a typo in one click)
(diff) ← Older revision | Latest revision (diff) | Newer revision → (diff)
Jump to navigation Jump to search

Template:TOC right

Motivation

Let G be an abelian group under addition. We can define a sort of multiplication on G by elements of by writing ng=g+g++gn for n+ and gG. We can extend this to the case where n is negative by writing (n)g=gggn. We would, however, like to be able to define a sort of multiplication of a group by an arbitrary ring.

Definition

Definition 1 (Module)
Let R be a ring and M an abelian group. We call M a left R-module if there is a function R×MM:(r,m)rm, called a scalar multiplication, satisfying
  1. (r+s)m=rm+sm,
  2. r(m+n)=rm+rn, and
  3. (rs)m=r(sm)
for all r,sR, m,nG.
We call R the ring of scalars of M.

Note: We can also define a right R-module analogously by using a function M×RM:(m,r)mr. In particular the third property then reads:

m(rs)=(mr)s

Note that the two notions coincide if R is a commutative ring, and in this case we can simply say that M is an R-module.

Definition 2: Given any ring R, we can define it's opposite ring, Rop, having the same elements and addition operation as R, but opposite multiplication. Their multiplication rules are related by rs=sr. In contrast to group theory, there is no reason in general for a ring to be isomorphic to its opposite ring.

The observant reader will have noticed that the scalar multiplication in a left R-module M is simply a ring homomorphism ϕ:REnd(M) such that rm=ϕ(r)(m) for all rR,mM. We leave it as an exercise to verify that the scalar multiplication in a right R-module is a ring homomorphism ϕ:RopEnd(M). Thus a right R-module is simply a left Rop-module. As a consequence of this, all the results we will formulate for left R-modules are automatically true for right R-modules as well. There are no assumptions that the module is unital, namely that 1m = m for all m in M.

Examples of Modules

  1. Any ring R is trivially an R-module over itself. More interestingly, any left ideal I of R is also a left R-module with the obvious scalar multiplication. In addition, if I is a two-sided ideal of R, then the quotient ring R/I is an R-module with the induced scalar multiplication r(s+I)=rs+I,(s+I)r=sr+I.
  2. If R is a ring, then the set Mn,m(R) of n×m matrices with entries in R is an R-module under componentwise addition and scalar multiplication. More generally, for any set X, the set RX of function from X to R, with or without finite support, is an R-module in an obvious way.
  3. The k-modules over a field k are simply the k-vector spaces.
  4. As was shown in the introduction of this chapter, any abelian group is a -module in a natural way. ("Natural" here has a rigorous mathematical meaning which will be explained later.
  5. Let S be a subring of a ring R. Then R is an S-module in a natural way. We can extend this as follows. Let S,R be rings and ϕ:SR a ring homomorphism. Then R is an S-module with scalar multiplication sr=ϕ(s)r and rs=rϕ(s) for all sS,rR.
  6. Any matrix ring of a ring R is a R-module under componentwise scalar multiplication.
  7. If S is a subring of a ring R, then any left R-module is also a left S-module with the restricted scalar multiplication. We will treat this more generally later.

Submodules

Definition 3: (Submodule)

Given a left R-module M a submodule of M is a subset NM satisfying
  1. N is a subgroup of M, and
  2. for all rR and all nN we have rnN.

The second condition above states that submodules are closed under left multiplication by elements of R; it is implicit that they inherit their multiplication from their containing module; R×NN must be the restriction of R×MM.

Example 4: Any module M is a submodule of itself, called the improper submodule, and the zero submodule consisting only of the additive identity of M, called the trivial submodule.

Example 5: A left ideal I is a submodule of R viewed as an S-module, where S is any (not necessarily proper) subring of R.

Lemma 6: Let M be a left R-module. Then the following are equivalent.

i) N is a submodule of M
ii) If riR and niN for all iI={1,,k},k, then iIriniN.
iii) If r1,r2R and n1,n2N, then r1n1+r2n2N.

Proof: i) => iii): r1n1 and r2n2 are in N by the second property, then r1n1+r2n2N by the first property of Definition 3.

iii) => ii): Follows by induction on k.

ii) => i): Let k=2, r1=1,r2=1, then for arbitrary n1,n2N be have n1n2N, proving N is a subgroup. Now let k=1, then for arbitrary r1,n1N, r1n1N, proving property 2 in Definition 3. Template:Unicode

The lemma gives an alternative characterisation of submodules, and those sets closed under linear combinations of elements.

Analogously to the case of vector spaces, we have ways of creating new subspaces from old ones. The rest of this subsection will be concerned with this.

Lemma 7: Let M be a left R-module, and let N and L be submodules of M. Then NL is a submodule in M, and it is the largest submodule contained in both N in L.

Proof: Let a,bNL and r,sR. Then ra+sbN and ra+sbL since N and L are submodules, so ra+sbNL and NL is a submodule of M. Now, assume that S is a submodule of M contained in N and L. Then any aS must be in both N and L and therefore in NL such that SNL, proving the lemma. Template:Unicode

Now, as the reader should expect at this point, given submodules N and L of M, the union NL is in general not a submodule. In fact, we have the following lemma:

Lemma 8: Let M be a left R-module and let N and L be submodules. Then NL is a submodule if and only if LN or NL.

Proof: The left implication is obvious. For the right implication, assume NL is a submodule of M. Then if nN and lL, then n+lNL, which implies that n+lM or n+lL. Assume without loss of generality that n+lN. Then, since N is a submodule, we must have (n+l)n=lN, proving LN. Template:Unicode

Definition 9: Let M be a left R-module, and let Ni be submodules for 1ik. Then define their sum, i=1kNi={j=1knj:njNj}.

Definition 9 has a straightforward extension to sums over arbitrary index sets. This definition is left for the reader to state. We will only need the finite case in this chapter.

Lemma 10: Let M be a left R-module and let N and L be submodules. Then N+L is a submodule of M, and it is the smallest submodule containing both N and L.

Proof: It is straightforward to see that N+L is a submodule. To see that it is the smallest submodule containing both N and L, let S be a submodule containing both N and L. Then for any nNS and lLS, we must have n+lS. But this is the same as saying that N+LS, proving the lemma. Template:Unicode

With Lemma 7 and Lemma 10 established, we can state the main result of this subsection.

Definition 11: Let M be a left R-module. Then let 𝒮(M) be the set of submodules ordered by set inclusion.

Lemma 12: Let M be a left R-module. Then 𝒮(M) forms a lattice, the join of N,L𝒮(M) being given by NL=N+L and their meet by NL=NL.

Proof: Most of the work is already done. All that remains is to check assosiativity, the absorption axioms and the idempotency axioms. The associativity is trivially satisfied, A(BC)=(AB)C and (A+B)+C=A+(B+C) for all A,B,C𝒮(M). As for absorption, We have to check A+(BA)=A and A(A+B)=A for all A,B𝒮(M), but this is also trivially true. Lastly, we obviously have A+A=A and AA=A for all 𝒮(M), so we are done. Template:Unicode

Corollary 13: Let M be a left R-module. Then 𝒮(M) is a modular lattice.

Note: Recall that 𝒮(M) is modular if and only if whenever A,B,C𝒮(M) such that AC, we have A+(BC)=(A+B)C.

Proof: Let aA,bB,cC such that a+b=c. Since AC, we have a=c for some cC, such that bC. Thus bBC and a+bA+(BC). On the other hand, we have a+bA+B and a+b=cC, so a+b(A+B)C. Template:Unicode

Definition 14: Let M be a left R-module. A submodule N is called maximal if whenever L is a submodule satisfying NLM, then L=N or L=M.

Theorem 15: Every submodule of a finitely generated left R-module is contained in a maximal submodule.

Proof: Let N be a submodule, and let S={L𝒮(M)|NLM}. Then S is a poset under set inclusion. Let {U1,U2,} be a chain in S, and note that U=U1+U2+ is a submodule containing each Ui, such that U is an upper bound for the chain. Then, since each chain in S has an upper bound, by Zorn's Lemma S has a maximal element, P, say. P is obviously an ideal containing N. By the definition of S, P is also a maximal submodule of M, proving the theorem. Template:Unicode

Generating Modules

Given a subset A of a left R-module M, we define the left submodule generated by A to be the smallest submodule (w.r.t. set containment) of M that contains A. It is denoted by RA for a reason which will become clear in a moment.

The existence of such a submodule comes from the fact that an intersection of R-modules is again an R-module: Consider the set S of all submodules of M containing A. Since M contains A, we see that S is non-empty. The intersection of the modules in S clearly contains A and is a submodule of M. Further, any submodule of M containing A also contains the intersection. Thus RA=S.

Assuming that M is unitary, the elements of RA have a simple description;

RA={i=1nriain,riR,aiA}.

That is, every element of RA can be written as a finite left linear combination of elements of A. This equality can be justified by double inclusion: First, any submodule containing A must contain all left R-linear combinations of elements of A since modules are closed under addition and left multiplication by elements of R. Thus, RA{i=1nriain,riR,aiA}. Secondly, the set of all such linear combinations forms a submodule of M containing A (use n=1 and r1=1R) and hence it contains RA.

Generating Submodules by Ideals

Consider any ring R, left ideal IR, and left R-module M. One can think of I as a subring of R (non-unitary when IR) and hence M is an I-module using the regular multiplication by elements of R.

If we consider the set IM={i=1nrimin,riI,miM} we obtain a submodule of M. This follows from our discussion of generated submodules. However, since I is not unitary, it is not necessary that IM=M.

Thus, we may consider the quotient module M/IM. Clearly this is an R-module but it is also an R/I module under the obvious action.

Proposition
Given an R-module M and ideal I of R, the Rmodule M/IM is an R/I-module with multiplication (r+I)(m+IM)=rm+IM.
proof.
To show that this is well defined, we observe that if r+I=s+I then rsI and hence
(rm+IM)(sm+IM)=rmsm+IM=(rs)m+IM=0+IM
since (rs)mIM. Thus,
(r+I)(m+IM)=rm+IM=sm+IM=(s+I)(m+IM)
which proves that the action of R/I on M/IM is well defined. It follows now that M/IM is an R/I-module simply because it is an R-module.

Quotient Modules

Recall that any subgroup N of an abelian group M allows one to construct an equivalence relation; for m,mM,

mmmmN.

Cosets of N, equivalence classes under the relation above, can then be endowed with a group structure, derived from the original group, and is given the name M/N. The sum of two cosets m+N=[m] and m+N=[m] is simply (m+m)+N=[m+m].

Lemma 16 Let M be a left R-module and N be a submodule. Then M/N, defined above, is a left R-module.

Proof: M/N is obviously an abelian group, so we just have to check that it has a well-defined R-action. Let rR and mM. Then we define r(m+N)=rm+N. The distributivity and associativity properties of the action are inherited from M, so we just need well-definedness. Let m,mM with mmN. Then r(mm+N)=r(mm)+N=N since N is a submodule, and we are done. Template:Unicode

Module Homomorphisms

Like all algebraic structures, we can define maps between modules that preserve their algebraic operations.

Definition (Module Homomorphism)
An R-module homomorphism ϕ:MN is a function from M to N satisfying
  1. ϕ(m+m)=ϕ(m)+ϕ(m) (it is a group homomorphism), and
  2. ϕ(rm)=rϕ(m).

When a map between two algebraic structures satisfies these two properties then it called an R-linear map.

Definition (Kernel, Image)
Given a module homomorphism ϕ:MN the kernel of ϕ is the set
kerϕ={mMϕ(m)=0}
and the image of ϕ is the set
ϕ(M)={nNmM,ϕ(m)=n}.

The kernel of ϕ is the set of elements in the domain that are sent to zero by ϕ. In fact, the kernel of any module homomorphism is a submodule of M. It is clearly a subgroup, from group theory, and it is also closed under multiplication by elements of R: ϕ(rm)=rϕ(m)=r(0)=0 for mkerϕ.

Similarly, one can show that the image of ϕ is a submodule of N.

Template:Subject

ja:加群