Girish Mahajan (Editor)

Proofs involving the Moore–Penrose pseudoinverse

Updated on
Edit
Like
Comment
Share on FacebookTweet on TwitterShare on LinkedInShare on Reddit

Let A be an m-by-n matrix over a field K , where K , is either the field R , of real numbers or the field C , of complex numbers. Then there is a unique n-by-m matrix A + over K , such that:

Contents

  1. A A+A = A
  2. A+A A+ = A+
  3. (AA+)* = AA+
  4. (A+A)* = A+A

A+ is called the Moore-Penrose pseudoinverse of A. Notice that A is also the Moore-Penrose pseudoinverse of A+ . That is, (A+ )+ = A.

Useful lemmas

These results are used in the proofs below. In the following lemmas, A is a matrix with complex elements and n columns, B is a matrix with complex elements and n rows.

Lemma 1: A*A = 0 ⇒ A = 0

The assumption says that all elements of A*A are zero. Therefore,

0 = Tr ( A A ) = j = 1 n ( A A ) j j = j = 1 n i = 1 m ( A ) j i A i j = i = 1 m j = 1 n | A i j | 2 .

Therefore, all A i j equal 0 i.e. A=0.

Lemma 3: ABB* = 0 ⇒ AB = 0

This is proved in a manner similar to the argument of Lemma 2 (or by simply taking the Hermitian conjugate).

Proof of uniqueness

Suppose that B and C are two n-by-m matrices over K satisfying the Moore-Penrose criteria. Observe then that

    AB = (AB)* = B*A* = B*(ACA)* = B*A*C*A* = (AB)*(AC)* = ABAC = AC.

Analogously we conclude that BA=CA. The proof is completed by observing that then

    B = BAB = BAC = CAC = C.

Proof of existence

The proof proceeds in stages.

1-by-1 matrices

For any x K , we define x + := { x 1 , if  x 0 0 , if  x = 0

It is easy to see that x + is a pseudoinverse of x (interpreted as a 1-by-1 matrix).

Square diagonal matrices

Let D be an n-by-n matrix over K with zeros off the diagonal. We define D + as an n-by-n matrix over K with ( D + ) i j := ( D i j ) + as defined above. We write simply D i j + for ( D + ) i j = ( D i j ) + .

Notice that D + is also a matrix with zeros off the diagonal.

We now show that D + is a pseudoinverse of D :

  1. ( D D + D ) i j = D i j D i j + D i j = D i j D D + D = D
  2. ( D + D D + ) i j = D i j + D i j D i j + = D i j + D + D D + = D +
  3. ( D D + ) i j = ( D D + ) j i ¯ = D j i D j i + ¯ = ( D j i D j i + ) = D j i D j i + = D i j D i j + ( D D + ) = D D +
  4. ( D + D ) i j = ( D + D ) j i ¯ = D j i + D j i ¯ = ( D j i + D j i ) = D j i + D j i = D i j + D i j ( D + D ) = D + D

Arbitrary matrices

The singular value decomposition theorem states that there exists a factorization of the form

A = U Σ V

where:

U is an m-by-m unitary matrix over K. Σ is an m-by-n matrix over K with nonnegative real numbers on the diagonal and zeros off the diagonal. V is an n-by-n unitary matrix over K.

Define A + as V Σ + U .

We now show that A + is a pseudoinverse of A :

  1. A A + A = U Σ V V Σ + U U Σ V = U Σ Σ + Σ V = U Σ V = A
  2. A + A A + = V Σ + U U Σ V V Σ + U = V Σ + Σ Σ + U = V Σ + U = A +
  3. ( A A + ) = ( U Σ V V Σ + U ) = ( U Σ Σ + U ) = U ( Σ Σ + ) U = U ( Σ Σ + ) U = U Σ V V Σ + U = A A +
  4. ( A + A ) = ( V Σ + U U Σ V ) = ( V Σ + Σ V ) = V ( Σ + Σ ) V = V ( Σ + Σ ) V = V Σ + U U Σ V = A + A

A*+=A+*

The proof works by showing that A+* satisfies the four criteria for the pseudoinverse of A*. Since this amounts to just substitution, it is not shown here.

The proof of this relation is given as Exercise 1.18c in.

A+ = A+ A+* A*

A+ = A+AA+ and AA+ = (AA+)* imply that A+ = A+(A A+)* = A+A+*A*.

A+ = A* A+* A+

A+ = A+AA+ and A+A = (A+A)* imply that A+ = (A+A)*A+ = A*A+*A+.

A = A+* A* A

A = A A+ A and A A+ = (A A+)* imply that A = (A A+)* A = A+* A* A.

A = A A* A+*

A = A A+ A and A+ A = (A+ A)* imply that A = A (A+ A)* = A A* A+*.

A* = A* A A+

This is the conjugate transpose of A = A+* A* A above.

A* = A+ A A*

This is the conjugate transpose of A = A A* A+* above.

Reduction to the Hermitian case

The results of this section show that the computation of the pseudoinverse is reducible to its construction in the Hermitian case. It suffices to show that the putative constructions satisfy the defining criteria.

A+ = A* (A A*)+

This relation is given as exercise 18(d) in, for the reader to prove, "for every matrix A". Write D = A* (A A*)+. Observe that

Similarly, (AA*)+AA*(AA*)+ = (AA*)+ implies that A*(AA*)+AA*(AA*)+ = A*(AA*)+ i.e. DAD = D.

Additionally, AD = AA*(AA*)+ so AD = (AD)*.

Finally, DA = A*(AA*)+A implies that (DA)* = A* ((AA*)+)*A = A* ((AA*)+)A = DA.

Therefore D = A+.

A+ = (A* A)+A*

This is proved in an analogous manner to the case above, using Lemma 2 instead of Lemma 3.

Products

For the first three proofs, we consider products C = AB.

A has orthonormal columns

If A has orthonormal columns i.e. A*A = I then A+=A*. Write D=B+A+ = B+A*. We show that D satisfies the Moore-Penrose criteria.

CDC = ABB+A*AB = ABB+B = AB = C .

DCD = B+A*ABB+A* = B+BB+A* = B+A* = D

(CD)* = D*B*A* = A(B+)*B*A* = A(BB+)*A* = ABB+A* = CD

(DC)* = B*A*D* = B*A*A(B+)* = (B+B)* = B+B = B+A*AB = DC

Therefore D = C+

B has orthonormal rows

If B has orthonormal rows i.e. BB* = I then B+=B*. Write D=B+A+ = B*A+. We show that D satisfies the Moore-Penrose criteria.

CDC = ABB*A+AB = AA+AB = AB = C .

DCD = B*A+ABB*A+ = B*A+AA+ = B*A+ = D

(CD)* = D*B*A* = (A+)*BB*A* = (A+)*A* = (AA+)* = AA+ = ABB*A+ = CD

(DC)* = B*A*D* = B*A*(A+)*B = B*(A+A)*B = B*A+AB = DC

Therefore D = C+

A has full column rank and B has full row rank

Since A has full column rank, A*A is invertible so (A*A)+ = (A*A)−1. Similarly, since B has full row rank, BB* is invertible so (BB*)+ = (BB*)−1.

Write D = B+A+ = B*(BB*)−1(A*A)−1A*. We show that D satisfies the Moore-Penrose criteria.

CDC = ABB*(BB*)−1(A*A)−1A*AB = AB = C .

DCD = B*(BB*)−1(A*A)−1A*ABB*(BB*)−1(A*A)−1A*= B*(BB*)−1(A*A)−1A* = D

CD = ABB*(BB*)−1(A*A)−1A* = A(A*A)−1A* = (A(A*A)−1A*)*(CD)* = CD.

DC = B*(BB*)−1(A*A)−1A*AB = B*(BB*)−1B = (B*(BB*)−1B)*(DC)* = DC.

Therefore D = C+

Conjugate transpose

Here, B = A , and thus C = A A and D = A + A + . We show that indeed D satisfies the four Moore-Penrose criteria.

Therefore D = C + . In other words:

and, since ( A ) = A

Projectors and subspaces

Define P = AA+ and Q = A+A. Observe that P2 = AA+AA+ = AA+ = P. Similarly Q2 = Q, and finally, P = P* and Q = Q*. Thus P and Q are orthogonal projection operators. Orthogonality follows from the relations P = P* and Q = Q*. Indeed, consider the operator P: any vector decomposes as

    x = Px + (I-P)x

and for all vectors x and y satisfying Px = x and (I-P)y = y, we have

    x*y = (Px)*(I-P)y = x*P*(I-P)y = x*P(I-P)y = 0.

It follows that PA = AA+A = A and A+P = A+AA+ = A+. Similarly, QA+ = A+ and AQ = A. The orthogonal components are now readily identified.

If y belongs to the range of A then for some x, y = Ax and Py = PAx = Ax = y. Conversely, if Py = y then y = AA+y so that y belongs to the range of A. It follows that P is the orthogonal projector onto the range of A. I - P is then the orthogonal projector onto the orthogonal complement of the range of A, which equals the kernel of A*.

A similar argument using the relation Q A* = A* establishes that Q is the orthogonal projector onto the range of A* and (I-Q) is the orthogonal projector onto the kernel of A.

Using the relations P(A+)* = P*(A+)* = (A+P)* = (A+)* and P = P* = (A+)*A* it follows that the range of P equals the range of (A+)*, which in turn implies that the range of I-P equals the kernel of A+. Similarly QA+ = A+ implies that the range of Q equals the range of A+. Therefore, we find,

Ker ( A + ) = Ker ( A ) . Im ( A + ) = Im ( A ) .

Least-squares minimization

In the general case, it is shown here for any m × n matrix A that A x b 2 A z b 2 where z = A + b . This lower bound need not be zero as the system A x = b may not have a solution (e.g. when the matrix A does not have full rank or the system is overdetermined).

To prove this, we first note that (stating the complex case), using the fact that P = A A + satisfies P A = A and P = P , we have

A ( A z b ) = A ( A A + b b ) = A ( P b b ) = A P b A b = ( P A ) b A b = 0

so that

A x b 2 2 = A z b 2 2 + ( A ( x z ) ) ( A z b ) + c.c. + A ( x z ) 2 2 = A z b 2 2 + ( x z ) A ( A z b ) + c.c. + A ( x z ) 2 2 = A z b 2 2 + A ( x z ) 2 2 A z b 2 2

as claimed.

If A is injective i.e. one-to-one (which implies m n ), then the bound is attained uniquely at z .

Minimum-norm solution to a linear system

The proof above also shows that if the system A x = b is satisfiable i.e. has a solution, then necessarily z = A + b is a solution (not necessarily unique). We show here that z is the smallest such solution (its Euclidean norm is uniquely minimum).

To see this, note first, with Q = A + A , that Q z = A + A A + b = A + b = z and that Q = Q . Therefore, assuming that A x = b , we have

z ( x z ) = ( Q z ) ( x z ) = z Q ( x z ) = z ( A + A x z ) = z ( A + b z ) = 0.

Thus

x 2 2 = z 2 2 + 2 z ( x z ) + x z 2 2 = z 2 2 + x z 2 2 z 2 2

with equality if and only if x = z , as was to be shown.

References

Proofs involving the Moore–Penrose pseudoinverse Wikipedia