AAMathNote

Polar Decomposition

Yun-Hao Lee, Cheng-Han Huang

Credit: Magda Ehlers from Pexels


1. Introduction

A polar decomposition says that an n × n matrix A n×n can be factorized into U|A| where |A| = (AA)1 2 and A = A¯T denotes the conjugate transpose of A.

2. Definitions and Statement

Definition 2.1 (Unitary matrix). A complex matrix U is unitary if and only if U = U1. In other words,

UU = UU = UU1 = I,the identity matrix

Definition 2.2 (Hermitian matrix). A complex matrix H is Hermitian if and only if H = H = H¯T .

Definition 2.3 (Positive semi-definite matrix). An n × n Hermitian complex matrix A is called positive semidefinite, denoted by A 0, if xT Ax 0 for every x n.

Theorem 2.4. For any complex n × n matrix A

A = U|A| = U(AA)1 2 ,whereUis ann × nunitary matrix.

Lemma 2.5. Let M be an n × n Hermitian matrix. M is positive semidefinite if and only if it can be decomposed as a product M = BB.

Proof. : If M = BB, then xMx = (xB)(Bx) = ||Bx||2 0 so M is positive definite.
: Suppose M is positive semidefinite, then M must be a Hermitian matrix and can be expressed in the form U1DU where U is unitary and D is diagonal (it is a theorem but we omit it for now). Moreover, M is positive semidefinite, the eigenvalues are nonnegative, we can therefore construct D1 2 by square rooting each elements of D, so D1 2 is also a diagonal matrix and (D1 2 )2 = D. Then

M = U1DU = UD1 2 D1 2 U = (UD1 2 )(D1 2 U) = BB

Lemma 2.6. A is unitary if and only if column vectors of A are orthogonal.

Proof. : Let A = [a1,a2,,an] be an n × n unitary matrix, by definition of unitary matrix,

In = AA = ( a1 a2 a n ) ( a1 a2 an )

then ai,aj = δij, the Kronecker delta, for all i,j. Hence the column vectors of A are orthogonal.
: Since the column vectors of A are orthogonal, then

δi,j = ai,ajand ( a1 a2 a n ) ( a1 a2 an ) = AAI n = AA

3. Proof

Now we proof the polar decomposition.

Proof. Case 1: If AA = diag[λ1,λ2,,λn], where

diag[λ1,λ2,,λn] = ( λ1 λ2 λ n ) ,a diagonal matrix.

Note that AA is a Hermitian matrix since (AA) = A(A) = AA.
Since AA is Hermitian matrix, AA is positive semidefinite by lemma 2.5, then λj 0 for all 1 j n. Suppose that λ1 λ2 λk > 0, k n, and λj = 0 for all k + 1 j n.
Without loss of generality, let

A = ( a1 a2 an ) A = ( a1¯T a2¯T an¯T ) ( λ1 λ2 λ k 0 0 ) = AA = ( a1,a1¯ an,a1¯ a1,an¯ an,an¯ ) {||ai,j|| = λj,for all1 j k aj = 0,for allk + 1 j n ai,aj = 0for allij { a1 λ1, a2 λ2,, ak λk}is orthonormal.

Extend it to orthonormal basis in n, that is, { a1 λ1, a2 λ2,, ak λk,uk+1,,un}.
Let U = [ a1 λ1, a2 λ2,, ak λk,uk+1,,un], by lemma 2.6, U is unitary and

U|A| = ( a1 λ1 a2 λ2 ak λk uk+1 un ) ( λ1 λ2 λk 0 0 ) = ( a1 a2 ak 0 0 ) = A

Case 2: For any complex matrix A, AA is a Hermitian matrix, then

AA = V ( λ1 λ2 λ n ) V where V  is unitary andλj 0for all1 j n

So

( λ1 λ2 λ n ) = V AAV = (V AV )(V AV ) = (A)(A),whereA = V AV

Since

|A| = V ( λ1 λ2 λn ) V |A| = ( λ1 λ2 λn ) = V |A|V

By Case 1, we have A = U|A|, where U is unitary, hence

V AV = UV |A|V A = V UV |A|

Note that if A,B are unitary, then AB is unitary since (AB)AB = BAAB = I.


Reference:

  • Beauregard, R. A., & Fraleigh, J. B. (1973). Linear Algebra: Pearson New International Edition. Pearson Education Limited.

Copyright© 2022 - AAMathNote
Powered by w3.css