Probability Practice Problems With Solutions 6
Probability Practice Problems With Solutions 6
TERMINOLOGY : The sum of the diagonal elements of a square matrix A is called the
trace of A, written tr(A), that is, for An×n = (aij ),
n
X
tr(A) = aii .
i=1
Result MAR6.1.
1. tr(A ± B) = tr(A) ± tr(B)
2. tr(cA) = ctr(A)
3. tr(A0 ) = tr(A)
4. tr(AB) = tr(BA)
Result MAR6.2.
1. |A0 | = |A|
2. |AB| = |BA|
3. |A−1 | = |A|−1
REVIEW : The table below summarizes equivalent conditions for the existence of an
inverse matrix A−1 (where A has dimension n × n).
PAGE 1
STAT 714 MATRIX ALGEBRA REVIEW 6
If u 6= 0, then A − λI must be singular (see last table). Thus, the values of λ which
satisfy Au = λu are those values where
|A − λI| = 0.
Aui = λi ui ,
From our discussion on systems of equations and consistency, we know a general solution
for ui is given by ui = [I − (A − λi I)− (A − λi I)]z, for z ∈ Rn .
Result MAR6.4. If A is a symmetric matrix, then there exists a basis for C(A) con-
sisting of eigenvectors of nonzero eigenvalues. If λ is a nonzero eigenvalue of multiplicity
m, then the basis will contain m eigenvectors for λ. Furthermore, N (A) consists of the
eigenvectors associated with λ = 0 (along with 0).
PAGE 2
STAT 714 MATRIX ALGEBRA REVIEW 6
Qn
1. |A| = i=1 λi
Pn
2. tr(A) = i=1 λi .
Result MAR6.6. Suppose that A is symmetric. The rank of A equals the number of
nonzero eigenvalues of A.
Proof. Write A in its spectral decomposition A = QDQ0 . Because r(D) = r(A) and
because the only nonzero elements in D are the nonzero eigenvalues, the rank of D must
be the number of nonzero eigenvalues of A.
showing that dim[N (A)] = n − r. Since A has n eigenvalues, all are accountedPfor λ = 1
(with multiplicity r) and for λ = 0 (with multiplicity n − r). Now tr(A) = i λi = r,
the multiplicity of λ = 1. But r(A) = dim[C(A)] = r as well.
PAGE 3
STAT 714 MATRIX ALGEBRA REVIEW 6
UPSHOT : In working with quadratic forms, we can, without loss of generality, assume
that the matrix of the quadratic form is symmetric.
1. A pd =⇒ |A| > 0
2. A nnd =⇒ |A| ≥ 0.
PAGE 4
STAT 714 MATRIX ALGEBRA REVIEW 6
the columns of A are linearly dependent; i.e., there exists an x 6= 0 such that Ax = 0.
Thus, A0 A is nnd but not pd, so it must be psd.
RESULT : A square matrix A is pd iff there exists a nonsingular lower triangular matrix
L such that A = LL0 . This is called the Choleski Factorization of A. Monahan
proves this result (see pp 258), provides an algorithm on how to find L, and includes an
example.
RESULT : Suppose that A is symmetric and pd. Writing A in its Spectral Decompo-
sition, we have A = QDQ0 . Because A is pd, λ1 , λ2 , ..., √
λn , the
√ eigenvalues
√ of A, are
1/2 0
positive. If we define A = QD Q , where D = diag( λ1 , λ2 , ..., λn ), then A1/2
1/2 1/2
is symmetric and
The matrix A1/2 is called the symmetric square root of A. See Monahan (pp 259-60)
for an example.
PAGE 5