Chapter 2 Fields and Vector Spaces

2.1 Fields

Definition 2.1 A field is a set F together with binary operations on F, which we will refer to as addition and multiplication, such that:

  • F together with addition is an abelian group (we use the notation a+b, 0 or 0F, a), and
  • F×:=F{0} together with multiplication is an abelian group (we use the notation ab or ab, 1, a1),
and such that the following axiom holds:
Distributivity: For all a,b,cF we have a(b+c)=ab+ac in F.

Example 2.2

  1. The sets Q,R and C with the usual addition and multiplication are fields (see also 1.2(b)).

  2. The set Z with the usual addition and multiplication is not a field because for instance there is no multiplicative inverse of 2 in Z.

  3. The set F2:={0,1} together with the following operations is a field. +0100111001000101 Note that 1+1=2 in Q but 1+1=0 in F2. F2 is the smallest field.

Proof (that F2 is a field): F2 with “+”, and F2{0}={1} with “”, are abelian groups (see 1.5(a)).
  Distributivity: We need to check a(b+c)=ab+ac for all a,b,cF2.
    First case: a=0 LHS =0, RHS =0+0=0.
    Second case: a=1 LHS =b+c= RHS.  

  1. (without proof) Let p be a prime. The set Fp :={¯0,¯1,,¯p1} together with the addition defined in Example 1.5(b) and the following multiplication is a field: ¯x¯y:=¯remainder left when xy is divided by p. (Why does this not work when p is not a prime, e.g. if p=4?)

Proposition 2.3 Let F be a field. Then:

  1. For all aF we have 0a=0.
  2. For all a,bF we have (a)b=(ab).

Proof. (a) We have 0+0a=0a=(0+0)a=0a+0a  (0 is neutral for “+” and by distributivity)
   0=0a.  (cancel 0a on both sides using 1.4(a))

  1. We have ab+(a)b=(a+(a))b  (by distributivity)
        =0b  (by definition of the additive inverse)
        =0  (by part (a))
    (a)b is the additive inverse of ab, i.e. (a)b=(ab).  

2.2 Vector spaces

Definition 2.4 Let F be a field. A vector space over F is an abelian group V (we will use “+” for the binary operation) together with a map F×VV (called scalar multiplication and written as (a,x)ax), such that the following axioms are satisfied:

  1. 1st distributivity law: For all a,bF and xV we have (a+b)x=ax+bx in V.
  2. 2nd distributivity law: For all aF and x,yV we have a(x+y)=ax+ay in V.
  3. For all a,bF and for all xV we have (ab)x=a(bx) in V.
  4. For all xV we have 1x=x in V.

The elements of V are called vectors. The elements of F will be referred to as scalars. We write 0F and 0V for the neutral elements of F and V, respectively, and often just 0 for both (when it is clear from the context if it is a scalar or a vector). Furthermore we use the notation uv for u+(v) when u,v are both vectors, or both scalars.

Example 2.5

  1. For every nN the set Rn together with the usual addition and scalar multiplication (as seen in Linear Algebra I) is a vector space over R. Similarly, for any field F, the set Fn:={(a1,,an): a1,,anF} together with component-wise addition and the obvious scalar multiplication is a vector space over F. For example F22={(0,0),(0,1),(1,0),(1,1)} is a vector space over F2; F=F1 is a vector space over F, and finally F0:={0} is a vector space over F.

  2. Let V be the additive group of C. We view the usual multiplication R×VV, (a,x)ax, as scalar multiplication of R on V. Then V is a vector space over R. Similarly, we can think of C or R as vector spaces over Q.

  3. Let V denote the abelian group R (with the usual addition). For aR and xV we put ax:=a2xV; this defines a scalar multiplication R×VV,(a,x)ax, of the field R on V. Which of the vector space axioms (see 2.4) hold for V with this scalar multiplication?

Solution:

  1. We need to check whether (a+b)x=ax+bx for all a,bR and xV.
    LHS =(a+b)2x; RHS =a2x+b2x=(a2+b2)x
    For a=1,b=1 and x=1 we have LHS RHS.
    First distributivity law does not hold.

  2. We need to check whether a(x+y)=ax+ay for all aR and x,yV.
    LHS=a2(x+y)RHS=a2x+a2y=a2(x+y)}LHS=RHS
    Second distributivity law does hold.

  3. We need to check whether a(bx)=(ab)x for all a,bR and xV.
    LHS=a(b2x)=a2(b2x)RHS=(ab)2x=(a2b2)x=a2(b2x)}LHS=RHS
    Axiom (iii) does hold.

  4. We have 1x=12x=x for all xV.
    Axiom (iv) does hold.

Proposition 2.6 Let V be a vector space over a field F and let a,bF and x,yV. Then we have:

  1. (ab)x=axbx
  2. a(xy)=axay
  3. ax=0Va=0F or x=0V
  4. (1)x=x

Proof: (a) (ab)x+bx=((ab)+b)x  (by first distributivity law)
          =(a+((b)+b))x=(a+0F)x=ax  (using field axioms)
      (ab)x=axbx.  (add bx to both sides)

  1. On Coursework.

  2. ”: On Coursework.
    ”: Put a=b and x=y in (a) and (b), respectively.

  3. Put a=0 and b=1 in (a) and use (c).  

The next example is the “mother” of almost all vector spaces. It vastly generalises the fourth of the following five ways of representing vectors and vector addition in R3.

  1. a_=(2.5,0,1)b_=(1,1,0.5)a_+b_=(3.5,1,0.5)

  2. a_=(1232.501)b_=(123110.5)a_+b_=(1233.510.5)

  3. a_:{1,2,3}Rb_:{1,2,3}Ra_+b_:{1,2,3}R12.51113.52021213130.530.5

Example 2.7 Let S be any set and let F be a field. Let FS:={f:SF} denote the set of all maps from S to F. We define an addition on FS and a scalar multiplication of F on FS as follows: When f,gFS and aF we set: (f+g)(s):=f(s)+g(s)for any sS(af)(s):=af(s)for any sS. Then FS is a vector space over F (see below for the proof).

Special Cases:

  1. Let S={1,,n}. Identifying any map f:{1,,n}F with the corresponding tuple (f(1),,f(n)), we see that FS can be identified with the set Fn of all n-tuples (a1,,an) considered in Example 2.5(a).

  2. Let S={1,,n}×{1,,m}. Identifying any map f:{1,,n}×{1,,m}F with the corresponding matrix: (f((1,1))f((1,m))f((n,1))f((n,m))) we see that FS can be identified with the set Mn×m(F) of (n×m)-matrices (a11a1man1anm) with entries in F. In particular Mn×m(F) is a vector space over F.

  3. Let S=N. Identifying any map f:NF with the sequence (f(1),f(2),f(3),) we see that FN can be identified with the set of all infinite sequences (a1,a2,a3,) in F.

  4. Let F=R and let S be an interval I in R. Then FS=RI is the set of all functions f:IR. (We can visualise these functions via their graph, similarly as in (V) above.)

Proof (that FS is a vector space over F): First, FS with the above defined “+” is an abelian group:

Associativity: Let f,g,hFS.
We need to show: (f+g)+h=f+(g+h) in FS
     ((f+g)+h)(s)=(f+(g+h))(s) for all sS.
LHS=(f+g)(s)+h(s)=(f(s)+g(s))+h(s)RHS=f(s)+(g+h)(s)=f(s)+(g(s)+h(s)}  (by definition of addition in FS)
LHS = RHS  (by associativity in F)

Identity element: Let 0_ denote the constant function SF,s0F.
For any fFS and sS we have (f+0_)(s)=f(s)+0_(s)=f(s)+0F=f(s), hence f+0_=f.
Similarly we have 0_+f=f.  (using definitions of 0_ and “+”, and field axioms)
0_ is the identity element.

Inverses: Let fFS. Define (f)(s):=f(s).
For any sS we have (f+(f))(s)=f(s)+(f)(s)=f(s)+(f(s))=0F=0_(s).
f+(f)=0_ in FS, so f is the inverse to f.  ( defns of “+”, “f”, 0_, and field axioms)

Commutativity: Let f,gFS.
For any sS we have (f+g)(s)=f(s)+g(s)=g(s)+f(s)=(g+f)(s).
f+g=g+f.  ( by the definition of “+”, and commutativity of + in F)

Now the four axioms from Definition 2.4 (only (i) and (iii) spelled out here, the others are similar):

First distributivity law: Let a,bF and fFS. We want to check that (a+b)f=af+bf:
For all sS we have
((a+b)f)(s)=(a+b)(f(s))  (by definition of the scalar multiplication)
     =a(f(s))+b(f(s))  (by distributivity in F)
     =(af)(s)+(bf)(s)  (by definition of the scalar multiplication)
     =(af+bf)(s)  (by definition of addition in FS)
(a+b)f=af+bf.

Axiom (iii): Let a,bF and fFS. We want to check that (ab)f=a(bf).
For all sS we have
((ab)f)(s)=(ab)(f(s))  (by definition of scalar multiplication in FS)
     =a(b(f(s)))  (by associativity of multiplication in F)
     =a((bf)(s))  (by definition of scalar multiplication in FS)
     =(a(bf))(s)  (by definition of scalar multiplication in FS)
(ab)f=a(bf).  

2.3 Subspaces

Definition 2.8 Let V be a vector space over a field F. A subset W of V is called a subspace of V if the following conditions hold:

  1. 0VW.
  2. W is closed under addition”: for all x,yW we also have x+yW.
  3. W is closed under scalar multiplication”: for all aF and xW we have axW.

Note that condition (b) states that the restriction of the addition in V to W gives a binary operation W×WW on W (addition in W). Similarly, condition (c) states that the scalar multiplication of F on V yields a map F×WW which we view as a scalar multiplication of F on W.

Proposition 2.9 Let V be a vector space over a field F and let W be a subspace of V. Then W together with the above mentioned addition and scalar multiplication is a vector space over F.

Proof: The following axioms hold for W because they already hold for V:

  • associativity of addition;
  • commutativity of addition;
  • all the four axioms in Definition 2.4.

There exists an additive identity element in W by condition 2.8(a) (i.e. 0W:=0VW).
It remains to show that additive inverses exist: Let xW. Then x=(1)x (see 2.6(d)) is in W by condition 2.8(c); and x satisfies x+(x)=0W=0V because it does so in V.  

Example 2.10

  1. Examples of subspaces of Rn as seen in Linear Algebra I, such as the nullspace of any real (n×m)-matrix, or the column space of any real (m×n)-matrix.

  2. The set of convergent sequences is a subspace of the vector space RN of all sequences (a1,a2,a3,) in R. A subspace of this subspace (and hence of RN) is the set of all sequences in R that converge to 0. (See Calculus I for proofs).

  3. Let AMl×m(R). Then W:={BMm×n(R)AB=0_} is a subspace of Mm×n(R).
    Proof:

    1. We have A0_=0_0_W.
    2. Let B1,B2W
      A(B1+B2)=AB1+AB2=0_+0_=0_
      B1+B2W.
    3. Let aR and BW
      A(aB)=a(AB)=a0_=0_
      aBW.  
  4. Let I be a non-empty interval in R. The following subsets of the vector space RI consisting of all functions from I to R are subspaces:

    1. For any s0I the subset W:={fRI:f(s0)=0} of RI.
      Proof:
      1. The zero function 0_ vanishes at s00_W.
      2. Let f,gW
        (f+g)(s0)=f(s0)+g(s0)=0+0=0
        f+gW.
      3. Let aR and fW
        (af)(s0)=af(s0)=a0=0
        afW.  
    2. The set of all continuous functions f:IR (see Calculus I).
    3. The set of all differentiable functions f:IR (see Calculus I).
    4. For any nN, the set Pn of polynomial functions f:IR of degree at most n, is a subspace by 3.2(c) and 3.3. A function f:IR is a polynomial function of degree at most n if there exists a0,,anR such that: f(s)=a0+a1s++ansn for all sI. Denoting the function IR,ssm, by tm, this means that f=a0t0+a1t1++antn as elements of the vector space RI. (We will also use the more natural notation 1 for t0, and t for t1.)
    5. The space of solutions of a homogeneous linear differential equation (without further explanation); e.g.: Pn={fRI:f is differentiable (n+1) times and f(n+1)=0_}
  5. The subset Zn of the vector space Rn over R is closed under addition but not closed under scalar multiplication: For instance, (1,0,,0)Zn and 12R, but 12(1,0,,0)Zn.

  6. The subsets W1:={(a,0):aR} and W2:={(0,b):bR} are subspaces of R2. The subset W:=W1W2 of the vector space R2 is closed under scalar multiplication but not under addition because, for instance, (1,0) and (0,1) are in W but (1,0)+(0,1)=(1,1)W.

Proposition 2.11 Let W1,W2 be subspaces of a vector space V over a field F. Then the intersection W1W2 and the sum of subspaces W1+W2:={x1+x2Vx1W1, x2W2} are subspaces of V as well.

Proof: For W1W2:

  1. We have 0VW1 and 0VW2  (because W1 and W2 are subspaces)
    0VW1W2.  (by definition of intersection)
  2. Let x,yW1W2
    x,yW1 and x,yW2  (by definition of intersection)
    x+yW1 and x+yW2  (because W1 and W2 are subspaces)
    x+yW1W2.  (by definition of intersection)
  3. Let aF and xW1W2
    xW1 and xW2  (by definition of intersection)
    axW1 and axW2  (because W1 and W2 are subspaces)
    axW1W2.  (by definition of intersection)

For W1+W2:

  1. We have 0V=0V+0VW1+W2.
  2. Let x,yW1+W2
    x1,y1W1 and x2,y2W2 with x=x1+x2, y=y1+y2  (by definition of W1+W2)
    x+y=(x1+x2)+(y1+y2)=
          =(x1+y1)+(x2+y2)W1+W2.  (because W1 and W2 are subspaces)
  3. Let aF and xW1+W2
    x1W1, x2W2 such that x=x1+x2  (by definition of W1+W2)
    ax=a(x1+x2)=ax1+ax2W1+W2.  (because W1 and W2 are subspaces)

Example 2.12 Let W1 and W2 be as in 2.10(f). Then W1+W2=R2.