Lecture 02_Several variables calculus
Lecture 02_Several variables calculus
Contents
1
2
1.1. Euclidean distance function. Here, we study Euclidean norm and distance
function in Rn . Euclidean space. Rn = {(x1 , x2 , . . . , xn )|xi ∈ R, 1 ≤ i ≤ n} is
called the n-dimensional Euclidean space when equipped with the Euclidean distance
function. In particular,
d(x, y) = (xi − yi )2 .
i=1
The pair (Rn , d)
is called the Euclidean space of dimension n. The distance function
d, defined above, is called Euclidean distance.
Note. The distance function d has the following fundamental properties:
1.2. Norm.
(1) Positive definiteness: kxk ≥ 0 for all x ∈ V , with equality if and only if
x = 0.
(2) Triangle inequality: kx + yk ≤ kxk + kyk, for all x, y ∈ V .
(3) Absolute homogeneity: kaxk = |a|kxk, for all a ∈ F and x ∈ V .
Exercise 1. Prove that the Euclidean norm satisfies all the properties in the defi-
nition of norm.
Proof. (1) The inequality kxk ≥ 0 follows from the fact that the sum of (finitely
many) non-negative reals is non-negative.
Now,
kxk = 0
⇐⇒ kxk2 = 0
⇐⇒ x21 + · · · + x2n = 0
⇐⇒ x1 = 0, . . . , xn = 0
⇐⇒ x = 0.
(2) Case 1: Suppose x and y are linearly dependent. Then it is straightforward to
see that equality holds. To see this, suppose x and y are linearly dependent,
which implies that
x = λy, or y = λx, for some λ ∈ R.
4
n
X n
X
xi yi = |λ| yi2
i=1 i=1
= |λ| × kyk2
= (|λ| × kyk) × kyk
= kλyk × kyk
= kxkkyk.
n
X
2
kλy − xk = (λyi − xi )2 > 0
i=1
n n n
! ! !
X X X
=⇒ λ2 yi2 − 2λ xi yi + x2i > 0.
i=1 i=1 i=1
n
!2 n
! n
!
X X X
4 xi yi −4 x2i yi2 <0
i=1 i=1 i=1
n
!2 n
! n
!
X X X
=⇒ x i yi < x2i yi2
i=1 i=1 i=1
n
!2
X
=⇒ x i yi < kxk2 kyk2 .
i=1
n
X
=⇒ xi yi < kxkkyk.
i=1
n
!1 n
!1
2 2
X 1 X
kaxk = (axi )2 = (a2 ) 2 x2i = |a| × kxk.
i=1 i=1
√
Note 1.3. Key definition used here is the following: For a ∈ R, we have a2 = |a|.
2. Inner Product
(1) Prove that T is norm preserving if and only if T is inner product preserving.
(2) Prove that such a linear transformation is 1 − 1 and T −1 is of the same sort.
haX, Y i = ahX, Y i
hX1 + X2 , Y i = hX1 , Y i + hX2 , Y i
Note. The key fact used here is the following: The multiplication of reals
is commutative, i.e., ab = ba, for all a, b ∈ R.
7
n
P n
P
(2) (a) haX, Y i = axi yi = a xi yi = ahX, Y i.
i=1 i=1
Now, we have
(c)
8
Exercise 5. If x, y ∈ Rn are nonzero, the angle between x and y, denoted by ∠(x, y),
is defined by
hx, yi
∠(x, y) = arc cos
kxkkyk
The linear transformation T is called angle preserving if
∠(T (x), T (y)) = ∠(x, y), ∀x, y ∈ Rn .
Exercise 6. Let h−, −i be an inner product and k·k be the norm induced by the
inner product on the vector space V . Prove that
ku + vk2 + ku − vk2 = 2(kuk2 + kvk2 ), for all u, v ∈ V.