Topics in Abstract Algebra/Linear algebra

From testwiki
Revision as of 01:22, 30 June 2023 by imported>Chumbigo (Minimum-norm solution to a linear system: Make computation steps simpler)
(diff) ← Older revision | Latest revision (diff) | Newer revision β†’ (diff)
Jump to navigation Jump to search

The Moore-Penrose inverse

Inverse matrices play a key role in linear algebra, and particularly in computations. However, only square matrices can possibly be invertible. This leads us to introduce the Moore-Penrose inverse of a potentially non-square real- or complex-valued matrix, which satisfies some but not necessarily all of the properties of an inverse matrix.

Definition.

Let A be an m-by-n matrix over a field 𝕂 and A+ be an n-by-m matrix over 𝕂, where 𝕂 is either ℝ, the real numbers, or β„‚, the complex numbers. Recall that A* refers to the conjugate transpose of A. Then the following four criteria are called the Moore–Penrose conditions for A:
  1. AA+A=A,
  2. A+AA+=A+,
  3. (AA+)*=AA+,
  4. (A+A)*=A+A.



We will see below that given a matrix A, there exists a unique matrix A+ that satisfies all four of the Moore–Penrose conditions. They generalise the properties of the usual inverse.

Remark.

If A is an invertible square matrix, then the ordinary inverse A1 satisfies the Moore-Penrose conditions for A. Observe also that if A+ satisfies the Moore-Penrose conditions for A, then A satisfies the Moore-Penrose conditions for A+.



Basic properties of the Hermitian conjugate

We assemble some basic properties of the conjugate transpose for later use. 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).

For any 𝕂-matrix A, A*A=0A=0


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

0=Tr(A*A)=j=1n(A*A)jj=j=1ni=1m(A*)jiAij=i=1mj=1n|Aij|2.

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

Lemma (2).

For any 𝕂-matrix A, A*AB=0AB=0


Proof. : 0=A*AB0=B*A*AB0=(AB)*(AB)0=AB(by Lemma 1)

Lemma (3).

For any 𝕂-matrix A, ABB*=0AB=0


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

Existence and uniqueness

We establish existence and uniqueness of the Moore-Penrose inverse for every matrix.

Theorem.

If A is a 𝕂-matrix and A1+ and A2+ satisfy the Moore-Penrose conditions for A, then A1+=A2+.


Proof. Let A be a matrix over ℝ or β„‚. Suppose that A1+ and A2+ are Moore–Penrose inverses of A. Observe then that

AA1+=(1)(AA2+A)A1+=(AA2+)(AA1+)=(3)(AA2+)*(AA1+)*=A2+*(AA1+A)*=(1)A2+*A*=(AA2+)*=(3)AA2+.

Analogously we conclude that A1+A=A2+A. The proof is completed by observing that then

A1+=(2)A1+AA1+=A1+AA2+=A2+AA2+=(2)A2+.


Theorem.

For every 𝕂-matrix A there is a matrix A+ satisfying the Moore-Penrose conditions for A


Proof. The proof proceeds in stages.

A is a 1-by-1 matrix

For any x𝕂, we define:

x+:={x1,if x00,if x=0

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

A is a square diagonal matrix

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

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

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

  1. (DD+D)ij=DijDij+Dij=DijDD+D=D
  2. (D+DD+)ij=Dij+DijDij+=Dij+D+DD+=D+
  3. (DD+)ij*=(DD+)ji=DjiDji+=(DjiDji+)*=DjiDji+=DijDij+(DD+)*=DD+
  4. (D+D)ij*=(D+D)ji=Dji+Dji=(Dji+Dji)*=Dji+Dji=Dij+Dij(D+D)*=D+D

A is a general diagonal matrix

Let D be an m-by-n matrix over 𝕂 with zeros off the main diagonal, where m and n are unequal. That is, Dij=di for some di𝕂 when i=j and Dij=0 otherwise.

Consider the case where n>m. Then we can rewrite D=[D0𝟎m×(nm)] by stacking where D0 is a square diagonal m-by-m matrix, and 𝟎m×(nm) is the m-by-(nβˆ’m) zero matrix. We define D+[D0+𝟎(nm)×m] as an n-by-m matrix over 𝕂, with D0+ the pseudoinverse of D0 defined above, and 𝟎(nm)×m the (nβˆ’m)-by-m zero matrix. We now show that D+ is a pseudoinverse of D:

  1. By multiplication of block matrices, DD+=D0D0++𝟎m×(nm)𝟎(nm)×m=D0D0+, so by property 1 for square diagonal matrices D0 proven in the previous section,DD+D=D0D0+[D0𝟎m×(nm)]=[D0D0+D0𝟎m×(nm)]=[D0𝟎m×(nm)]=D.
  2. Similarly, D+D=[D0+D0𝟎m×(nm)𝟎(nm)×m𝟎(nm)×(nm)], so D+DD+=[D0+D0𝟎m×(nm)𝟎(nm)×m𝟎(nm)×(nm)][D0+𝟎(nm)×m]=[D0+D0D0+𝟎(nm)×m]=D+.
  3. By 1 and property 3 for square diagonal matrices, (DD+)*=(D0D0+)*=D0D0+=DD+.
  4. By 2 and property 4 for square diagonal matrices, (D+D)*=[(D0+D0)*𝟎m×(nm)𝟎(nm)×m𝟎(nm)×(nm)]=[D0+D0𝟎m×(nm)𝟎(nm)×m𝟎(nm)×(nm)]=D+D.

Existence for D such that m>n follows by swapping the roles of D and D+ in the n>m case and using the fact that (D+)+=D.

A is an arbitrary matrix

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 𝕂.
Σ is an m-by-n matrix over 𝕂 with nonnegative real numbers on the diagonal and zeros off the diagonal.
V is an n-by-n unitary matrix over 𝕂.[1]

Define A+ as VΣ+U*.

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

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

This leads us to the natural definition:

Definition (Moore-Penrose inverse).

Let A be a 𝕂-matrix. Then the unique 𝕂-matrix satisfying the Moore-Penrose conditions for A is called the Moore-Penrose inverse A+ of A.



Basic properties

We have already seen above that the Moore-Penrose inverse generalises the classical inverse to potentially non-square matrices. We will now list some basic properties of its interaction with the Hermitian conjugate, leaving most of the proofs as exercises to the reader.

Exercise.

For any 𝕂-matrix A, A*+=A+*



The following identities hold:

  1. A+ = A+ A+* ATemplate:Sup
  2. A+ = ATemplate:Sup A+* A+
  3. A = A+* ATemplate:Sup A
  4. A = A ATemplate:Sup A+*
  5. ATemplate:Sup = ATemplate:Sup A A+
  6. ATemplate:Sup = A+ A ATemplate:Sup

Proof of the first one: A+=A+AA+ and AA+=(AA+)* imply that A+=A+(AA+)*=A+A+*A*. β–‘

The remaining identities are left as exercises.

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.

Proposition.

For every 𝕂-matrix A, A+=A*(AA*)+


Proof. Observe that

AA*=AA*(AA*)+AA*AA*=ADAA*0=(ADI)AA*0=ADAA(by Lemma 3)A=ADA

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+.

Exercise.

For every 𝕂-matrix A, A+=(A*A)+A*



Products

We now turn to calculating the Moore-Penrose inverse for a product of two matrices, C=AB.

Proposition.

If A has orthonormal columns i.e. A*A=I, then for any 𝕂-matrix B of the right dimensions, (AB)+=B+A+.


Proof. Since A*A=I, A+=A*. Write C=AB and D=B+A+=B+A*. We show that D satisfies the Moore–Penrose criteria for C.

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+.

Exercise.

If B has orthonormal rows, then for any 𝕂-matrix A of the right dimensions, (AB)+=B+A+.



Another important special case which approximates closely that of invertible matrices is when A has full column rank and B has full row rank.

Proposition.

If A has full column rank and B has full row rank, then (AB)+=B+A+.


Proof. 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*(using reduction to the Hermitian case). 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+.

We finally derive a formula for calculating the Moore-Penrose inverse of AA*.

Proposition.

If B=A*, then (AB)+=A+*A+.


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

CDC=AA*A+*A+AA*=A(A+A)*A+AA*=AA+AA+AA*=AA+AA*=AA*=CDCD=A+*A+AA*A+*A+=A+*A+A(A+A)*A+=A+*A+AA+AA+=A+*A+AA+=A+*A+=D(CD)*=(AA*A+*A+)*=A+*A+AA*=A+*(A+A)*A*=A+*A*A+*A*=(AA+)*(AA+)*=AA+AA+=A(A+A)*A+=AA*A+*A+=CD(DC)*=(A+*A+AA*)*=AA*A+*A+=A(A+A)*A+=AA+AA+=(AA+)*(AA+)*=A+*A*A+*A*=A+*(A+A)*A*=A+*A+AA*=DC

Therefore, D=C+. In other words:

(AA*)+=A+*A+

and, since (A*)*=A

(A*A)+=A+A+*

Projectors and subspaces

The defining feature of classical inverses is that AA1=A1A=I. What can we say about AA+ and A+A?

We can derive some properties easily from the more basic properties above:

Exercise.

Let A be a 𝕂-matrix. Then (AA+)2=(AA+),(A+A)2=(A+A),(AA+)*=(AA+) and (A+A)*=(A+A)



We can conclude that P=AA+ and Q=A+A are orthogonal projections.

Proposition.

Let A be a 𝕂-matrix. Then P=AA+ and Q=A+A are orthogonal projections


Proof. Indeed, consider the operator P: any vector decomposes as

x=Px+(IP)x

and for all vectors x and y satisfying Px=x and (IP)y=y, we have

x*y=(Px)*(IP)y=x*P*(IP)y=x*P(IP)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.

We finish our analysis by determining image and kernel of the mappings encoded by the Moore-Penrose inverse.

Proposition.

Let A be a 𝕂-matrix. Then Ker(A+)=Ker(A*) and Im(A+)=Im(A*).


Proof. 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. IP 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 QA*=A* establishes that Q is the orthogonal projector onto the range of A* and (IQ) 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 IP 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*).

Applications

We present two applications of the Moore-Penrose inverse in solving linear systems of equations.

Least-squares minimization

Moore-Penrose inverses can be used for least-squares minimisation of a system of equations that might not necessarily have an exact solution.

Proposition.

For any m×n matrix A, Axb2Azb2 where z=A+b.


Proof. We first note that (stating the complex case), using the fact that P=AA+ satisfies PA=A and P=P*, we have

A*(Azb)=A*(AA+bb)=A*(Pbb)=A*P*bA*b=(PA)*bA*b=0

so that (c.c. stands for the Hermitian conjugate of the previous term in the following)

Axb22=Azb22+(A(xz))*(Azb)+c.c.+A(xz)22=Azb22+(xz)*A*(Azb)+c.c.+A(xz)22=Azb22+A(xz)22Azb22

as claimed.

Remark.

This lower bound need not be zero as the system Ax=b may not have a solution (e.g. when the matrix A does not have full rank or the system is overdetermined). If A is injective i.e. one-to-one (which implies mn), then the bound is attained uniquely at z.



Minimum-norm solution to a linear system

The proof above also shows that if the system Ax=b is satisfiable i.e. has a solution, then necessarily z=A+b is a solution (not necessarily unique). We can say more:

Proposition.

If the system Ax=b is satisfiable, then z=A+b is the unique solution with smallest Euclidean norm.


Proof. Note first, with Q=A+A, that Qz=A+AA+b=A+b=z and that Q*=Q. Therefore, assuming that Ax=b, we have

z*(xz)=(Qz)*(xz)=z*Q(xz)=z*(A+Axz)=z*(A+bz)=0.

Thus

x22=z+(xz)22=z22+z*(xz)+z*(xz)+xz22=z22+xz22z22

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

An immediate consequence of this result is that z is also the uniquely smallest solution to the least-squares minimization problem for all Ax=b, including when A is neither injective nor surjective. It can be shown that the least-squares approximation Az=yb is unique. Thus it is necessary and sufficient for all x that solve the least-squares minimization to satisfy Ax=y=Az=AA+b. This system always has a solution (not necessarily unique) as Az lies in the column space of A. From the above result the smallest x which solves this system is A+(AA+b)=A+b=z.

Notes

Template:Reflist

References

Template:BookCat

  1. ↑ Some authors use slightly different dimensions for the factors. The two definitions are equivalent.