Exercise 20.9

Show that the euclidean metric d on n is a metric, as follows: If x,y n and c , define

x + y = (x1 + y1,,xn + yn), cx = (cx1,,cxn) , x y = x1y1 + + xnyn.
(a)
Show that x (y + z) = (x y) + (x z).
(b)
Show that |x y| x y. [Hint: If x,y0, let a = 1 x and b = 1 y, and use the fact that ax ± by 0.]
(c)
Show that x + y x + y. [Hint: Compute (x + y) (x + y) and apply (b).]
(d)
Verify that d is a metric.

Answers

First, we show some basic properties of these operations that will be useful:

Lemma 1. For any x,y n and a , we assert the following:

(1)
The dot product is commutative, that is x y = y x.
(2)
0 x = 0.
(3)
x = 0 if and only if x = 0.
(4)
x 0
(5)
x x = x2
(6)
ax = |a| x

Proof. For assertion (1) clearly

x y = i=1nx iyi = i=1ny ixi = y x

by the definition of the dot product. Regarding (2), we clearly have

0 x = i=1n0 x i = i=1n0 = 0.

For (3) first suppose that x0 so that that there is an i {1,,n} where xk0 so that clearly xk2 > 0. Then we have

x = i=1nx i2 = i=kxi2 + ikxi2 = x k2 + ikxi2 x k2 + 0 = x k2 > 0

since each term in the sum ikxi2 is non-negative so the overall sum is as well. Thus of course x0. This shows the forward implication by contrapositive. For the reverse direction, suppose that x = 0 so that

x = 0 = [ i=1n02] 12 = [ i=1n0]12 = [0]12 = 0.

Assertion (4) is fairly obvious from the definition. Clearly each xi2 0 since it is a square, so that i=1nxi2 0 as well. It then follows from Corollary 1 that

x = [ i=1nx i2] 12 012 = 0

as desired. Assertion (5) is also easy to show:

x x = i=1nx ixi = i=1nx i2 = ( [ i=1nx i2] 12) 2 = x2

by definition.

For part (6) we have by definition that

ax = [ i=1n(ax i)2] 12 = [ i=1na2x i2] 12 = [a2 i=1nx i2] 12 = [a2] 12 [ i=1nx i2] 12 = |a| x

as desired. □

Main Problem.

(a)

Proof. By definition, we have that

y + z = (y1 + z1,,yn + yn)

so that clearly

x (y + z) = i=1nx i(yi + zi) = i=1n(x iyi + xizi) = i=1nx iyi + i=1nx izi = (x y) + (x z)

as desired. □

(b)

Proof. First, if x = 0 then clearly by Lemma 1 parts (2) and (3)

|x y| = |0 y| = |0| = 0 0 = 0 y = 0 y = x y.

Similarly if y = 0 then by all parts of Lemma 1

|x y| = |x 0| = |0 x| = |0| = 0 0 = x0 = x 0 = x y.

So in what follows assume that x,y0. Then by Lemma 1 part (3) we have that x and y are both nonzero so that a = 1 x and b = 1 y are defined. Then, by Lemma 1 part (4), we of course have

ax ± by 0.

Since clearly

ax ± by = (ax1 ± by1,,axn ± byn)

by the definition of the operations, we have

[ i=1n(ax i ± byi)2] 12 = ax ± by 0.

It then follows from Lemma 1 that

i=1n(ax i ± byi)2 02 = 0 i=1n(a2x i2 ± 2abx iyi + b2y i2) 0 a2 i=1nx i2 ± 2ab i=1nx iyi + b2 i=1ny i2 0 a2 x2 ± 2ab(x y) + b2 y2 0 ± 2ab(x y) a2 x2 b2 y2 ± 2 x y x y x2 x2 y2 y2 ± 2 x y x y 1 1 ± 2 x y x y 2 x y x y.

Hence we have that both x y x y and x y x y so that x y x y. Hence

x y x y x y

so we can conclude that |x y| x y as desired. □

(c)

Proof. We have

x + y2 = (x + y) (x + y) (by Lemma 1  part (5)) = (x + y) x + (x + y) y (by part (a)) = x (x + y) + y (x + y) (by Lemma 1  part (1)) = x x + x y + y x + y y (by part (a)) = x2 + x y + y x + y2 (by Lemma 1  part (5)) = x2 + x y + x y + y2 (by Lemma 1  part (1)) x2 + x y + x y + y2 (by part (b)) = x2 + 2 x y + y2 = (x + y)2.

The desired result that x + y x + y then follows from Corollary 1. □

(d)

Proof. First recall that the euclidean metric on n is defined as

d(x,y) = x y.

Then part (1) of the definition of a metric follows directly from Lemma 1 since of course

d(x,y) = x y 0.

We also have that x = y if and only if x y = 0, which is true if and only if

d(x,y) = x y = 0

by Lemma 1 part (3). Similarly part (2) of the definition follows from Lemma 1 part (6) as follows:

d(x,y) = x y = (1)(y x) = |1| y x = y x = d(y,x).

Lastly, for part (3) of the definition, we have that

d(x,z) = x y = x z + y y = (x y) + (y z) x y + x z = d(x,y) + d(y,z),

where we have used what was shown in part (c). This shows that d has all the properties required to be a metric. □

User profile picture
2019-12-01 00:00
Comments