Vector product

The scalar product maps a pair of vectors to a scalar: Rn×RnR. The scalar product can be defined in the vector space Rn with any n. In contrast, the vector product (also known as the cross product), which maps a pair of vectors to another vector (Rn×RnRn) in the same vector space, can be defined only in the 3-dimensional space, R3.



Definition (Vector product)

Let a,bR3 be row vectors a=(a1,a2,a3) and b=(b1,b2,b3). Then their vector product (also called the cross product or outer product), denoted a×b, is the vector defined as

a×b=(a2b3a3b2,a3b1a1b3,a1b2a2b1).

Remark. Some authors prefer to denote the vector product by [a,b] rather than a×b. □

Let e1=(1,0,0),e2=(0,1,0),e3=(0,0,1), then the cross product may be formally expressed as a determinant as in

a×b=|e1e2e3a1a2a3b1b2b3|=|a2a3b2b3|e1|a1a3b1b3|e2+|a1a2b1b2|e3=(|a2a3b2b3|,|a1a3b1b3|,|a1a2b1b2|)=(a2b3a3b2,a3b1a1b3,a1b2a2b1).

Theorem 

Let a,bR3. Then we have the following.

  1. If a=0 or b=0, then a×b=0.
  2. If a and b are parallel, that is, a=λb or b=μa for some non-zero λ,μR, then a×b=0.
  3. a×b=(b×a). (Thus, the vector product is not commutative.)
  4. For any λR, λ(a×b)=(λa)×b=a×(λb).
  5.  e1×e2=e3, e2×e3=e1, e3×e1=e2.
Proof. (Exercise.) ■

In the following, the scalar product between a and b is denoted by ab rather than a,b. Recall that the scalar product is also called the dot product.

Definition (Triple product)

The triple product of three vectors a,b,cR3 is defined by
a(b×c).

Theorem

Let a,b,cR3 be row vectors. Their triple product is given by the determinant:
a(b×c)=|abc|.
Proof. Let a=(a1,a2,a3), b=(b1,b2,b3), c=(c1,c2,c3). By definition,
b×c=(b2c3b3c2,b3c1b1c3,b1c2b2c1)
so
a(b×c)=a1(b2c3b3c2)+a2(b3c1b1c3)+a3(b1c2b2c1)=a1|b2b3c2c3|a2|b1b3c1c3|+a3|b1b2c1c2|=|a1a2a3b1b2b3c1c2c3|=|abc|.

Corollary 

a(b×c)=c(a×b)=b(c×a).
Proof. By the property of determinants, we have
a(b×c)=|abc|=|cba|=|cab|=c(a×b).
The rest is similar. ■

Corollary 

a(a×b)=0.
Proof. (Exercise.) ■
Remark. Similarly, we have b(a×b)=0.
This result indicates that the vector product a×b is perpendicular to both a and b. If a×b0, the three vectors a, b and their vector product form a right-handed set. This means if your right index and middle fingers to directions of a and b, respectively, then your right thumb points to the direction of a×b. □

Corollary

a×(b+c)=a×b+a×c.
Proof. (Exercise.) ■

Lemma

Let a,bR3. If ab=0, then a×b=ab.
Proof. If a=0 or b=0, the result is trivial.
Suppose a,b0. Since ab=0, we have
a1b1+a2b2+a3b3=0.
Squaring both sides yields
a12b12+a22b22+a32b32+2a1a2b1b2+2a2a3b2b3+2a3a1b3b1=0.
so, in particular,
2a1a2b1b22a2a3b2b32a3a1b3b1=a12b12+a22b22+a32b32.
Using this, we compute 
a×b2=(a2b3a3b2)2+(a3b1a1b3)2+(a1b2a2b1)2=a22b32+a32b222a2a3b2b3+a32b12+a12b322a1a3b1b3+a12b22+a22b122a1a2b1b2=a22b32+a32b22+a32b12+a12b32+a12b22+a22b12+(a12b12+a22b22+a32b32)=(a12+a22+a32)(b12+b22+b32)=a2b2.
Remark. This lemma says that, if the vectors a and b are perpendicular to each other (including the case one (or both) of them is zero), then the length of their vector product is the product of their lengths. □

Theorem

Let a,bR3 such that the angle between them is θ. Then
a×b=ab|sinθ|.
Proof. Let a,bR3 be non-zero vectors, and let the angle between them be θ. So we have
ab=abcosθ.
Using the unit vector defined by
a^=1aa,
let us define
b=(a^b)a^
and
b=bb.
By this definition, we have
(eq:bbpp)b=b+b.
Clearly, b is parallel to a and
(eq:paracos)b2=(a^b)2=b2cos2θ.
On the other hand, b is perpendicular to a because
ba^=ba^(a^b)a^2=0.
It follows that bb=0. Therefore, from (eq:bbpp), we have
b2=b2+b2.
Substituting (eq:paracos), 
b2=b2b2cos2θ=b2sin2θ.
Hence
b=b|sinθ|.
Now consider the vector product a×b. Since a and b are parallel to each other, a×b=0. Therefore,
a×b=a×(b+b)=a×b+a×b=a×b.
Since ab=0 (i.e., they are perpendicular), using the above lemma,
a×b=ab=ab|sinθ|.
Remark. Note that any two vectors a and b define a parallelogram. That is, the origin and the position vectors a,b and a+b make the vertices of a parallelogram. You should prove that the area of this parallelogram is given by ab|sinθ| where θ is the angle between a and b. □

Remark. Similarly, any three vectors a,b and c can define a parallelepiped (a solid body of which each face is a parallelogram). We can show that the triple product a(b×c) corresponds to the signed volume of that parallelepiped. Here, the term ``signed'' indicates that this ``volume'' can be negative. More specifically, the sign of this volume is positive if the triple (a,b,c), in this order, makes a right-hand set, or negative if it makes a left-hand set. □

Comments

Popular posts from this blog

Birth process

Branching processes: Mean and variance

Informal introduction to formal logic