Norm and scalar product

 A vector space is a set with addition and scalar products. We can introduce more structures into this set. Here, we define a vector's norm (length) and the scalar product (dot product) between vectors.



Definition (Norm, length, modulus)

The norm (also called length or modulus) of the vector x=(x1,,xn) is the real number defined by

(eq:norm)x=i=1nxi2=x12+x22++xn2.

Remark. The norm of a vector, as defined above, is also known as the 2-norm or the Euclidean norm of the vector. More generally, for kN, the k-norm of the vector xRn is defined as

xk=i=1n|xi|kk.

Example. When n=1, the norm of x=(x1) is given by

x=x12=|x1|

which coincides with the absolute value of the real number x1.

When n=2, the norm of of x=(x1,x2) is

x=x12+x22

which is the distance between the origin and x=(x1,x2) in the 2-dimensional space. 

We can consider the modulus of a vector defined by (eq:norm) as a generalization of the distance between the origin and x in the n-dimensional space. □

Definition (Unit vector)

Let xRn. x is called a unit vector if x=1


We can define a ``multiplication'' between two vectors to obtain a scalar.

Definition (Scalar product)

Let x=(x1,,xn), y=(y1,,yn)Rn. The scalar product of these two vectors is defined by

x,y=i=1nxiyi=x1y1+x2y2++xnyn.

Remark. The scalar product is also called the inner product or dot product, and they can be denoted as xy or (x,y) or x|y. □

Remark. The scalar product may be considered as a map

,:Rn×RnR

that maps a pair of vectors to a real number. □

You should prove the following lemma.

Lemma

Let x,y,zRn and λR.
  1. x2=x,x.
  2. λx=|λ|x.
  3. x,y=y,x.
  4. x+y,z=x,z+y,z.
  5. x,y+z=x,y+x,z.
  6. λx,y=λx,y.
  7. λx,y=x,λy.
The next theorem provides a geometric interpretation of the scalar product.

Theorem (Angle between vectors in R2)

Suppose that u,vR2, then 

u,v=uvcosθ

where θ is the angle between the vectors u and v.

Proof. First, consider the case where u and v are unit vectors, namely, u=v=1.

Then we can write u=(u1,u2)=(cosϕ,sinϕ) and v=(v1,v2)=(cosψ,sinψ) where ϕ and ψ are angles of u and v from (1,0), respectively. Then

u,v=cosϕcosψ+sinϕsinψ=cos(ϕψ).

Note that ϕψ is the angle between u and v so that θ=ϕψ, and the claim holds.


Next, consider the general case where u and v are not unit vectors. We can write u=uu^ and v=vv^ where u^ and v^ are unit vectors. Thus,

u,v=uvu^,v^=uvcosθ

as required. ■

Remark. Let's look at this theorem from a different perspective. Recall that we constructed C from R2

See also: Constructing complex numbers.

So, a complex number is actually a vector in R2. The unit vector u corresponds to the complex number eiϕ, and the unit vector v corresponds to eiψ.

Note that the scalar product

u,v=(u1,u2),(v1,v2)=u1v1+u2v2

is the real part of 

(u1iu2)(v1+iv2)=(u1v1+u2v2)+i(u1v2u2v1),

which, in turn, is the real part of

eiϕeiψ=ei(ϕψ)=cos(ϕψ)isin(ϕψ).

We can prove the same theorem for R3 (You should try to prove it). We want the same result for any dimension, Rn. How do we prove that? No, we don't prove that. Instead, we define the angle between two vectors in terms of the scalar product. But before that, we need the following theorem.

Theorem (Cauchy-Schwarz inequality)

Let x,yRn. Then

|x,y|xy.

Proof. The result is trivial if x=0 or y=0.


Suppose x0 and y0. We have

x+λy20

for all λR since it's the square of a real number. Thus

x+λy,x+λy0.

Expanding the left-hand side using the properties of scalar product, we have

λ2y2+2λx,y+x20.

The left-hand side is a quadratic polynomial in λ with a positive coefficient of λ2. If this inequality should hold for any real value of λ, the discriminant of this quadratic polynomial should be non-positive:

4x,y24x2y20

which rearranges to

|x,y|xy.

The Cauchy-Schwarz inequality plays an important role in many fields in mathematics, including statistics.

Definition (Angle between two vectors in Rn)

Let x,yRn be non-zero vectors. The angle between x and y is defined to be that angle θ such that

cosθ=x,yxy.

From the Cauchy-Schwarz inequality, we can see that the right-hand side in the above definition is bounded between 1 and 1 so that we indeed have 1cosθ1 as it should be.

Theorem (Triangle inequality)

Let x,yRn. Then

x+yx+y.

Proof. We can use the Cauchy-Schwarz inequality to show the following.

x+y2=x+y,x+y=x2+2x,y+y2x2+2|x,y|+y2x2+2xy+y2=(x+y)2.

Comments

Popular posts from this blog

Birth process

Branching processes: Mean and variance

Informal introduction to formal logic