Skip to main content
Logo image

Section PEE Properties of Eigenvalues and Eigenvectors

The previous section introduced eigenvalues and eigenvectors, and concentrated on their existence and determination. This section will be more about theorems, and the various properties eigenvalues and eigenvectors enjoy. Like a good 4×100 meter relay, we will lead-off with one of our better theorems and save the very best for the anchor leg.

Subsection BPE Basic Properties of Eigenvalues

Proof.

We will establish by induction (Proof Technique I) that any set of k eigenvectors of A with distinct eigenvalues λ1,λ2,λ3,,λk is a linearly independent set. Suppose A has size n.
Base Case.
When k=1, {x1} is a set with a single nonzero vector and thus is linearly independent.
Induction Step.
Begin with a relation of linear dependence on the set {x1,x2,x3,,xk}
a1x1+a2x2+a3x3++akxk=0.
Then
0=(AλkIn)0Theorem MMZM=(AλkIn)(a1x1+a2x2+a3x3++akxk)Definition RLD=(AλkIn)a1x1++(AλkIn)akxkTheorem MMDAA=a1(AλkIn)x1++ak(AλkIn)xkTheorem MMSMM=a1(Ax1λkInx1)++ak(AxkλkInxk)Theorem MMDAA=a1(Ax1λkx1)++ak(Axkλkxk)Theorem MMIM=a1(λ1x1λkx1)++ak(λkxkλkxk)Definition EEM=a1(λ1λk)x1++ak(λkλk)xkProperty DSA=a1(λ1λk)x1++ak1(λk1λk)xk1+ak(0)xkProperty AICN=a1(λ1λk)x1++ak1(λk1λk)xk1+0Theorem ZSSM=a1(λ1λk)x1++ak1(λk1λk)xk1Property Z
This equation is a relation of linear dependence on the set {x1,x2,x3,,xk1}, which is a linearly independent set by the induction hypothesis. So the scalars must all be zero by Definition LI. That is, ai(λiλk)=0 for 1ik1. However, we have the hypothesis that the eigenvalues are distinct, so λiλk0 for 1ik1. So Theorem ZPZF implies ai=0 for 1ik1.
This reduces the original relation of linear dependence on {x1,x2,x3,,xk} to the simpler equation akxk=0. By Theorem SMEZV we conclude that ak=0 or xk=0. Eigenvectors are never the zero vector (Definition EEM), so ak=0. Now all of the scalars ai, 1ik are zero, and so the only relation of linear dependence on the set {x1,x2,x3,,xk} is trivial. So by Definition LI, the set {x1,x2,x3,,xk} is linearly independent.
The next theorem gives us a convenient upper limit on the number of eigenvalues.

Proof.

We argue by contradiction (Proof Technique CD). Assume that A has n+1 or more distinct eigenvalues. Then there is a set of n+1 or more eigenvectors of A, with distinct eigenvalues. This is a set of n+1 or more vectors from Cn that will be linearly independent by Theorem EDELI. But this contradicts Theorem MVSLD, so our assumption is false, and there are no more than n distinct eigenvalues.
Notice that once we have found n distinct eigenvalues for a matrix of size n, then we know there are no more eigenvalues. Example DEMS5 is an example, and the upcoming Theorem DED also considers this situation.
There is a simple connection between the eigenvalues of a matrix and whether or not the matrix is nonsingular.

Proof.

We have the following equivalences:
A is singularA0In is singularProperty ZM0 is an eigenvalue of ATheorem ESM.
With an equivalence about singular matrices we can update our list of equivalences about nonsingular matrices.

Proof.

The equivalence of the first and last statements is Theorem SMZE, reformulated by negating each statement in the equivalence. So we are able to improve on Theorem NME7 with this addition.

Sage NME8. Nonsingular Matrix Equivalences, Round 8.

Zero eigenvalues are another marker of singular matrices. We illustrate with two matrices, the first nonsingular, the second not.
Certain changes to a matrix change its eigenvalues in a predictable way.

Proof.

Let x0 be one eigenvector of A for λ. Then
(αA)x=α(Ax)Theorem MMSMM=α(λx)Definition EEM=(αλ)xProperty SMAC.
So x0 is an eigenvector of αA for the eigenvalue αλ.
Unfortunately, there are not parallel theorems about the sum or product of arbitrary matrices. But we can prove a similar result for powers of a matrix.

Proof.

Let x0 be one eigenvector of A for λ. Then we proceed by induction on s (Proof Technique I). First, for s=0, employing Theorem MMIM and Property OC to establish the base case,
Asx=A0x=Inx=x=1x=λ0x=λsx.
So λs is an eigenvalue of As in this special case. For the induction step, we assume the theorem is true for s, and find
As+1x=AsAx=As(λx)Definition EEM=λ(Asx)Theorem MMSMM=λ(λsx)Induction Hypothesis=(λλs)xProperty SMAC=λs+1x.
So x0 is an eigenvector of As+1 for λs+1, and induction tells us the theorem is true for all s0.
While we cannot prove that the sum of two arbitrary matrices behaves in any reasonable way with regard to eigenvalues, we can work with the sum of dissimilar powers of the same matrix. We have already seen that eigenvalues arise as roots of polynomials (Theorem EMRCP). A theme of this chapter is relationships between eigenvalues and polynomials, and our next theorem is the next component of this theme.

Proof.

Let x0 be one eigenvector of A for λ, and write q(x)=a0+a1x+a2x2++amxm. Then
q(A)x=(a0A0+a1A1+a2A2++amAm)x=(a0A0)x+(a1A1)x+(a2A2)x++(amAm)xTheorem MMDAA=a0(A0x)+a1(A1x)+a2(A2x)++am(Amx)Theorem MMSMM=a0(λ0x)+a1(λ1x)+a2(λ2x)++am(λmx)Theorem EOMP=(a0λ0)x+(a1λ1)x+(a2λ2)x++(amλm)xProperty SMAC=(a0λ0+a1λ1+a2λ2++amλm)xProperty DSAC=q(λ)x.
So x0 is an eigenvector of q(A) for the eigenvalue q(λ).
Inverses and transposes also behave predictably with regard to their eigenvalues.

Proof.

Notice that since A is assumed nonsingular, A1 exists by Theorem NI, but more importantly, λ1=1/λ does not involve division by zero since Theorem SMZE prohibits this possibility.
Let x0 be one eigenvector of A for λ. Suppose A has size n. Then
A1x=A1(1x)Property OC=A1(1λλx)Property MICN=1λA1(λx)Theorem MMSMM=1λA1(Ax)Definition EEM=1λ(A1A)xTheorem MMA=1λInxDefinition MI=1λxTheorem MMIM.
So x0 is an eigenvector of A1 for the eigenvalue 1λ.
The proofs of the theorems above have a similar style to them. They all begin by grabbing an eigenvalue-eigenvector pair and adjusting it in some way to reach the desired conclusion. You should add this to your toolkit as a general approach to proving theorems about eigenvalues.
So far we have been able to reserve the characteristic polynomial for strictly computational purposes. However, sometimes a theorem about eigenvalues can be proved easily by employing the characteristic polynomial (rather than using an eigenvalue-eigenvector pair). The next theorem is an example of this.

Proof.

Suppose A has size n. Then
pA(x)=det(AxIn)Definition CP=det((AxIn)t)Theorem DT=det(At(xIn)t)Theorem TMA=det(AtxInt)Theorem TMSM=det(AtxIn)Definition IM=pAt(x)Definition CP.
So A and At have the same characteristic polynomial, and by Theorem EMRCP, their eigenvalues are identical and have equal algebraic multiplicities. Notice that what we have proved here is a bit stronger than the stated conclusion in the theorem.
If a matrix has only real entries, then eigenvalues will arise as the roots of a polynomial with real coefficients. Complex numbers could result as roots of this polynomial, but they are roots of quadratic factors with real coefficients, and as such, come in conjugate pairs. The next theorem proves this, and a bit more, without ever mentioning a polynomial.

Proof.

We have
Ax=AxA has real entries=AxTheorem MMCC=λxDefinition EEM=λxTheorem CRSM.
So x is an eigenvector of A for the eigenvalue λ.
This phenomenon is amply illustrated in Example CEMS6, where the four complex eigenvalues come in two pairs, and the two basis vectors of the eigenspaces are complex conjugates of each other. Theorem ERMCP can be a time-saver for computing eigenvalues and eigenvectors of real matrices with complex eigenvalues, since the conjugate eigenvalue and eigenspace can be inferred from the theorem rather than computed.

Subsection ME Multiplicities of Eigenvalues

A polynomial of degree n will have exactly n roots. From this fact about polynomial equations we can say more about the algebraic multiplicities of eigenvalues.

Proof.

We will prove a more general result by induction (Proof Technique I). Then the theorem will be true as a special case. We will carefully state this result as a proposition indexed by m, m1.
P(m): Suppose that A is an m×m matrix whose entries are complex numbers or linear polynomials in the variable x of the form cx, where c is a complex number. Suppose further that there are exactly k entries that contain x and that no row or column contains more than one such entry. Then, when k=m, det(A) is a polynomial in x of degree m, with leading coefficient ±1, and when k<m, det(A) is a polynomial in x of degree k or less.
Base Case: Suppose A is a 1×1 matrix. Then its determinant is equal to the lone entry (Definition DM). When k=m=1, the entry is of the form cx, a polynomial in x of degree m=1 with leading coefficient 1. When k<m, then k=0 and the entry is simply a complex number, a polynomial of degree 0k. So P(1) is true.
Induction Step: Assume P(m) is true, and that A is an (m+1)×(m+1) matrix with k entries of the form cx. There are two cases to consider.
Suppose k=m+1. Then every row and every column will contain an entry of the form cx. Suppose that for the first row, this entry is in column t. Compute the determinant of A by an expansion about this first row (Definition DM). The term associated with entry t of this row will be of the form
(cx)(1)1+tdet(A(1|t)).
The submatrix A(1|t) is an m×m matrix with k=m terms of the form cx, no more than one per row or column. By the induction hypothesis, det(A(1|t)) will be a polynomial in x of degree m with coefficient ±1. So this entire term is then a polynomial of degree m+1 with leading coefficient ±1.
The remaining terms (which constitute the sum that is the determinant of A) are products of complex numbers from the first row with cofactors built from submatrices that lack the first row of A and lack some column of A, other than column t. As such, these submatrices are m×m matrices with k=m1<m entries of the form cx, no more than one per row or column. Applying the induction hypothesis, we see that these terms are polynomials in x of degree m1 or less. Adding the single term from the entry in column t with all these others, we see that det(A) is a polynomial in x of degree m+1 and leading coefficient ±1.
The second case occurs when k<m+1. Now there is a row of A that does not contain an entry of the form cx. We consider the determinant of A by expanding about this row (Theorem DER), whose entries are all complex numbers. The cofactors employed are built from submatrices that are m×m matrices with either k or k1 entries of the form cx, no more than one per row or column. In either case, km, and we can apply the induction hypothesis to see that the determinants computed for the cofactors are all polynomials of degree k or less. Summing these contributions to the determinant of A yields a polynomial in x of degree k or less, as desired.
Definition CP tells us that the characteristic polynomial of an n×n matrix is the determinant of a matrix having exactly n entries of the form cx, no more than one per row or column. As such we can apply P(n) to see that the characteristic polynomial has degree n.

Proof.

By the definition of the algebraic multiplicity (Definition AME), we can factor the characteristic polynomial as
pA(x)=c(xλ1)αA(λ1)(xλ2)αA(λ2)(xλ3)αA(λ3)(xλk)αA(λk)
where c is a nonzero constant. (We could prove that c=(1)n, but we do not need that specificity right now. See Exercise PEE.T30) The left-hand side is a polynomial of degree n by Theorem DCP and the right-hand side is a polynomial of degree i=1kαA(λi). So the equality of the polynomials’ degrees gives the equality i=1kαA(λi)=n.

Proof.

Since λ is an eigenvalue of A, there is an eigenvector of A for λ, x. Then xEA(λ), so γA(λ)1, since we can extend {x} into a basis of EA(λ) (Theorem ELIS).
To show γA(λ)αA(λ) is the most involved portion of this proof. To this end, let g=γA(λ) and let x1,x2,x3,,xg be a basis for the eigenspace of λ, EA(λ). Construct another ng vectors, y1,y2,y3,,yng, so that
{x1,x2,x3,,xg,y1,y2,y3,,yng}
is a basis of Cn. This can be done by repeated applications of Theorem ELIS.
Finally, define a matrix S by
S=[x1|x2|x3||xg|y1|y2|y3||yng]=[x1|x2|x3||xg|R]
where R is an n×(ng) matrix whose columns are y1,y2,y3,,yng. The columns of S are linearly independent by design, so S is nonsingular (Theorem NMLIC) and therefore invertible (Theorem NI).
Then
[e1|e2|e3||en]=In=S1S=S1[x1|x2|x3||xg|R]=[S1x1|S1x2|S1x3||S1xg|S1R].
So
(*)S1xi=ei1ig.
Preparations in place, we compute the characteristic polynomial of A,
pA(x)=det(AxIn)Definition CP=1det(AxIn)Property OCN=det(In)det(AxIn)Definition DM=det(S1S)det(AxIn)Definition MI=det(S1)det(S)det(AxIn)Theorem DRMM=det(S1)det(AxIn)det(S)Property CMCN=det(S1(AxIn)S)Theorem DRMM=det(S1ASS1xInS)Theorem MMDAA=det(S1ASxS1InS)Theorem MMSMM=det(S1ASxS1S)Theorem MMIM=det(S1ASxIn)Definition MI=pS1AS(x)Definition CP.
What can we learn then about the matrix S1AS?
S1AS=S1A[x1|x2|x3||xg|R]=S1[Ax1|Ax2|Ax3||Axg|AR]Definition MM=S1[λx1|λx2|λx3||λxg|AR]Definition EEM=[S1λx1|S1λx2|S1λx3||S1λxg|S1AR]Definition MM=[λS1x1|λS1x2|λS1x3||λS1xg|S1AR]Theorem MMSMM=[λe1|λe2|λe3||λeg|S1AR]S1S=In, (*) above
Now imagine computing the characteristic polynomial of A by computing the characteristic polynomial of S1AS using the form just obtained. The first g columns of S1AS are all zero, save for a λ on the diagonal. So if we compute the determinant by expanding about the first column, successively, we will get successive factors of (λx). More precisely, let T be the square matrix of size ng that is formed from the last ng rows and last ng columns of S1AR. Then
pA(x)=pS1AS(x)=(λx)gpT(x).
This says that (xλ) is a factor of the characteristic polynomial at least g times, so the algebraic multiplicity of λ as an eigenvalue of A is greater than or equal to g (Definition AME). In other words,
γA(λ)=gαA(λ)
as desired.
Theorem NEM says that the sum of the algebraic multiplicities for all the eigenvalues of A is equal to n. Since the algebraic multiplicity is a positive quantity, no single algebraic multiplicity can exceed n without the sum of all of the algebraic multiplicities doing the same.

Subsection EHM Eigenvalues of Hermitian Matrices

Recall that a matrix is Hermitian (or self-adjoint) if A=A (Definition HM). In the case where A is a matrix whose entries are all real numbers, being Hermitian is identical to being symmetric (Definition SYM). Keep this in mind as you read the next two theorems. Their hypotheses could be changed to “suppose A is a real symmetric matrix.”

Proof.

Let x0 be one eigenvector of A for the eigenvalue λ. Then
(λλ)x,x=λx,xλx,xProperty DCN=x,λxλx,xTheorem IPSM=x,AxAx,xDefinition EEM=Ax,xAx,xTheorem HMIP=0.
Since x0, by Theorem PIP we know x,x0. Then by Theorem ZPZF, λλ=0, and so λ=λ. If a complex number is equal to its conjugate, then it has a complex part equal to zero, and therefore is a real number.
Notice the key step of this proof is the ability to pitch a Hermitian matrix from one side of the inner product to the other.
Look back and compare Example ESMS4 and Example CEMS6. In Example CEMS6 the matrix has only real entries, yet the eigenvalues come as roots of polynomial that are complex numbers. However, in Example ESMS4, the matrix has only real entries, but is also symmetric, and hence Hermitian. So by Theorem HMRE, we were guaranteed eigenvalues that are real numbers.
In many physical problems, a matrix of interest will be real and symmetric, or Hermitian. Then if the eigenvalues are to represent physical quantities of interest, Theorem HMRE guarantees that these values will not be complex numbers.
The eigenvectors of a Hermitian matrix also enjoy a pleasing property that we will exploit later.

Proof.

Let x be an eigenvector of A for λ and let y be an eigenvector of A for a different eigenvalue ρ. So we have λρ0. Then
(λρ)x,y=λx,yρx,yProperty DCN=λx,yx,ρyTheorem IPSM=λx,yx,ρyTheorem HMRE=Ax,yx,AyDefinition EEM=Ax,yAx,yTheorem HMIP=0.
Because λ and ρ are presumed to be different, λρ0, and Theorem ZPZF implies that x,y=0. In other words, x and y are orthogonal vectors according to Definition OV.
Notice again how the key step in this proof is the fundamental property of a Hermitian matrix (Theorem HMIP) — the ability to swap A across the two arguments of the inner product. Notice too, that we can always apply the Gram-Schmidt procedure (Theorem GSP) to any basis of any eigenspace, along with scaling the resulting the orthogonal vectors by their norm to arrive at an orthonormal basis of the eigenspace. For a Hermitian matrix, pairs of eigenvectors from different eigenspaces are also orthogonal. If we dumped all these basis vectors into one big set it would be an orthonormal set. We will build on these results and continue to see some more interesting properties in Section OD.

Reading Questions PEE Reading Questions

1. Eigenvalues of a Nonsingular Matrix.

How can you identify a nonsingular matrix just by looking at its eigenvalues?

2. Maximum Number of Distinct Eigenvalues.

How many different eigenvalues may a square matrix of size n have?

3. Eigenvalues of a Hermitian Matrix.

What is amazing about the eigenvalues of a Hermitian matrix and why is it amazing?

Exercises PEE Exercises

M20.

This exercise will show we can use a polynomial to convert one matrix into another, with predictable changes in its eigenvalues. In Example ESMS4 the 4×4 symmetric matrix
C=[1011011111101101]
is shown to have the three eigenvalues λ=3,1,1. Suppose we wanted a 4×4 matrix that has the three eigenvalues λ=4,0,2. We can employ Theorem EPM by finding a polynomial that converts 3 to 4, 1 to 0, and 1 to 2. Such a polynomial is called an interpolating polynomial, and in this example we can use
r(x)=14(x2+4x5)=14x2+x54.
(a)
Verify that the polynomial r(x) converts the eigenvalues as advertised.
Solution.
We will not discuss how to concoct the interpolating polynomial, r(x), but a text on numerical analysis should provide the details. For now, it should be routine to verify that r(3)=4, r(1)=0 and r(1)=2.
(b)
In the style of Example PM, compute the matrix r(C).
Solution.
Now compute
r(C)=14C2+C54I4=14[3222232222322223]+[1011011111101101]54[1000010000100001]=12[1133113333113311].
(c)
Compute the eigenvalues of r(C) directly and verify that they are as expected.
Solution.
notice that the multiplicities are the same, and the eigenspaces of C and r(C) are identical.

T10.

Suppose that A is a square matrix. Prove that the constant term of the characteristic polynomial of A is equal to the determinant of A.
Solution.
Suppose that the characteristic polynomial of A is
pA(x)=a0+a1x+a2x2++anxn.
Then
a0=a0+a1(0)+a2(0)2++an(0)n=pA(0)=det(A0In)Definition CP=det(A).

T20.

Suppose that A is a square matrix. Prove that a single vector may not be an eigenvector of A for two different eigenvalues.
Solution.
Suppose that the vector x0 is an eigenvector of A for the two eigenvalues λ and ρ, where λρ. Then λρ0, and we also have
0=AxAxProperty AIC=λxρxDefinition EEM=(λρ)xProperty DSAC.
By Theorem SMEZV, either λρ=0 or x=0, which are both contradictions.

T21.

Suppose that A is a square matrix of size n with an eigenvalue λ. For αC, prove that λ+α is an eigenvalue of the matrix A+αIn.
  1. Construct a proof that begins by employing a vector x that is an eigenvector of A for λ.
  2. Construct a proof that establishes that λ+α is a root of the characteristic polynomial of A+αIn.

T22.

Suppose that U is a unitary matrix with eigenvalue λ. Prove that λ has modulus 1, i.e. |λ|=1. This says that all of the eigenvalues of a unitary matrix lie on the unit circle of the complex plane.

T30.

Theorem DCP tells us that the characteristic polynomial of a square matrix of size n has degree n. By suitably augmenting the proof of Theorem DCP prove that the coefficient of xn in the characteristic polynomial is (1)n.

T50.

Theorem EIM says that if λ is an eigenvalue of the nonsingular matrix A, then 1λ is an eigenvalue of A1. Write an alternate proof of this theorem using the characteristic polynomial and without making reference to an eigenvector of A for λ.
Solution.
Since λ is an eigenvalue of a nonsingular matrix, λ0 (Theorem SMZE). A is invertible (Theorem NI), and so λA is invertible (Theorem MISM). Thus λA is nonsingular (Theorem NI) and det(λA)0 (Theorem SMZD). We have
pA1(1λ)=det(A11λIn)Definition CP=1det(A11λIn)Property OCN=1det(λA)det(λA)det(A11λIn)Property MICN=1det(λA)det((λA)(A11λIn))Theorem DRMM=1det(λA)det(λAA1(λA)1λIn)Theorem MMDAA=1det(λA)det(λIn(λA)1λIn)Definition MI=1det(λA)det(λIn+λ1λAIn)Theorem MMSMM=1det(λA)det(λIn+1AIn)Property MICN=1det(λA)det(λIn+AIn)Property OCN=1det(λA)det(λIn+A)Theorem MMIM=1det(λA)det(AλIn)Property ACM=1det(λA)pA(λ)Definition CP=1det(λA)0Theorem EMRCP=0Property ZCN.
So 1λ is a root of the characteristic polynomial of A1 and so is an eigenvalue of A1. This proof is due to Sara Bucht.
You have attempted 1 of 4 activities on this page.