Numerical computation of the Complex Eigenpair of a Large...

24
Numerical computation of the Complex Eigenpair of a Large Sparse Matrix R. O . . Akino . la and A. Spence 23rd March 2016

Transcript of Numerical computation of the Complex Eigenpair of a Large...

Page 1: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Numerical computation of theComplex Eigenpair of a Large

Sparse Matrix

R. O. . Akino. la and A. Spence

23rd March 2016

Page 2: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Let A ∈ Rn×n be a large, sparse, nonsymmetricmatrix.B ∈ Rn×n, Symmetric Positive Definite (SPD)matrix.We consider the problem of computing theeigenpair (z,λ) from the GeneralisedEigenvalue Problem

Az = λBz, z ∈ Cn, z 6= 0, (1)

where λ ∈ C is the eigenvalue.We assume that the eigenpair of interest (z,λ)is algebraically simple. The left e-vector ψ is 3

Page 3: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

ψHBz 6= 0. (2)

By adding the normalisation

zHBz = 1, (3)

to (1) & v = [zT ,λ],

F(v) =[

(A− λB)z−1

2zHBz + 12

]= 0. (4)

Page 4: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Lemma

z̄ in zHBz = z̄T Bz is not differentiable.

Proof.

If z = x + iy , z̄ = x − iy , then the Cauchy-Riemannequations are not satisfied. u(x , y) = x ,v(x , y) = −y , then ux (x , y) = 1 and vy (x , y) = −1,whereas the Cauchy-Riemann equations requirethat ux (x , y) = vy (x , y).

Newton’s method cannot be applied to (4).

Page 5: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

For a real eigenpair (z,λ), Newton’s method forsolving (4) involves the solution of the (n + 1)square linear systems[

A− λ(k)B −Bz(k)

−(Bz(k))T 0

] [∆z(k)

∆λ(k)

]=

[−(A− λ(k)B)z(k)

12z(k)

TBz(k) − 1

2

],

(5)for real unknowns ∆v(k) = [∆z(k)

T,∆λ(k)].

Update v(k+1) = v(k) + ∆v(k),for k = 0,1,2, · · · .

Page 6: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Ruhe (1973) added the normalization cHz = 1,c is a fixed complex vector instead of zHBz = 1.Parlett and Saad (1987) studied inverseiteration with a fixed complex shift. Numericalexamples showed linear convergence to theeigenvalue closest to the shift.Tisseur (2001) used the normalization eT

s z = 1Both Ruhe’s and Tisseur’s normalizations aredifferentiable, but we use the naturalnormalization for the eigenvector.

Page 7: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

z = z1 + iz2 and λ = α + iβ. (1), (4) becomes

F(v) =

(A− αB)z1 + βBz2−βBz1 + (A− αB)z2−1

2(zT1 Bz1 + zT

2 Bz2) +12

= 0. (6)

The Jacobian, with v = [z1, z2, α, β]T is

Fv(v) =

(A− αB) βB −Bz1 Bz2−βB (A− αB) −Bz2 −Bz1−(Bz1)

T −(Bz2)T 0 0

.

(7)

Page 8: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Let

w =

[z1z2

], w1 =

[z2−z1

]. (8)

We define the real 2n by 2n matrix M as

M =

[(A− αB) βB−βB (A− αB)

]. (9)

Also, we form the 2n by 2 real matrix

N =

[−Bz1 Bz2−Bz2 −Bz1

]=[−B2w B2w1

], (10)

where B2 =

[B OO B

].

Page 9: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Note that because at the root,[(A− αB) βB−βB (A− αB)

] [z1z2

]=

[(A− αB)z1 + βBz2(A− αB)z2 − βBz1

]= 0.

In the same vein, we find[(A− αB) βB−βB (A− αB)

] [z2−z1

]= 0.

The Jacobian (7) can be rewritten in partitionedform

Fv =

[M −B2w B2w1

−(B2w)T 0 0

]=

[M N

−(B2w)T 0T

].

(11)

Page 10: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

For all ψ ∈ N(A− λB)H\{0}, we defineψ = ψ1 + iψ2, where ψ1,ψ2 ∈ Rn,

ψH(A− λB) = (ψT1 − iψT

2 )[(A− αB)− iβB]

= ψT1 (A− αB)− βψT

2 B

− i [βψT1 B + ψT

2 (A− αB)] = 0T .

[ψT1 ψT

2 ]M = [ψT1 ψT

2 ]

[(A− αB) βB−βB (A− αB)

]= 0T

[ψT1 , ψT

2 ] is a left nullvector of M. Similarly,

[ψT2 −ψT

1 ]M = [ψT2 −ψT

1 ]

[(A− αB) βB−βB (A− αB)

]= 0T .

Page 11: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

C =

[ψ1 ψ2ψ2 −ψ1

]. (12)

Now, observe that the condition (2), implies

ψHBz = [ψT1 Bz1 +ψT

2 Bz2]+ i [ψT1 Bz2−ψT

2 Bz1] 6= 0.

Theorem

Assume that the eigenpair (z,λ) of the pencil (A,B)is algebraically simple. If z1 and z2 are nonzerovectors, then φ = {τ[zT

2 ,−zT1 ,0,0], τ ∈ R} is the

eigenspace corresponding to the zero eigenvalue ofFv(v) at the root.

Page 12: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Proof

Post-multiply Fv(v) by the unknown nonzero vectorφ = [p′,q′]T and H = CT N[

M N−(B2w)T 0T

] [p′

q′

]= 0.

Mp′ + Nq′ = 0 (13)

wT B2p′ = 0. (14)

H =

[ψT

1 ψT2

ψT2 −ψT

1

] [−Bz1 Bz2−Bz2 −Bz1

]=

[−(ψT

1 Bz1 + ψT2 Bz2) ψT

1 Bz2 −ψT2 Bz1

ψT1 Bz2 −ψT

2 Bz1 (ψT1 Bz1 + ψT

2 Bz2)

].

Page 13: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

CT Mp′ + CT Nq′ = 0. (15)

But, CT M = 0T . Consequently, CT Nq′ = 0, or

Hq′ = CT Nq′

=

[−(ψT

1 Bz1 + ψT2 Bz2) ψT

1 Bz2 −ψT2 Bz1

ψT1 Bz2 −ψT

2 Bz1 (ψT1 Bz1 + ψT

2 Bz2)

]q′

= 0.

Now, det H 6= 0. H is nonsingular. Thus, q′ = 0.Equation (13) now becomes Mp′ = 0, meaning thatp′ ∈ N(M), p′ = µw + τw1. From (14),

0 = wT B2p′ = µwT B2w + τwT B2w1.

wT B2w1 = 0 and wT B2w 6= 0, µ = 0 and sop′ = τw1. Hence, for all

Page 14: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

τ ∈ R\{0}, p′ = [τz2,−τz1]T ∈ N(M) also satisfies

equation (14). φ = τ[z2,−z1,0,0]T as the onlynonzero nullvector of Fv(v).

Corollary

If the eigenpair (z,λ) of (A,B) is algebraicallysimple, then the Jacobian Fv(v) in (11) is of full rankat the root.

Proof.

The theorem above guarantees the existence of asingle nonzero nullvector of Fv(v) at the root, thenrank

(Fv(v)

)= 2n + 1. Therefore, the Jacobian (7)

is of full rank at the root. (Dimension theorem).

Page 15: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Eigenpair Computation using Gauss-Newton’smethod

A,B, v(0) = [z(0)1 , z(0)2 , α(0), β(0)]T , kmax and tol.for k = 0,1,2, . . . , until convergence

Find the reduced QR factorisation ofFv(v(k))T = QR.Solve RT g(k) = −F(v(k)) for g(k) in (7).Compute ∆v(k) = Qg(k) for ∆v(k) using (6).Update v(k+1) = v(k) + ∆v(k).v(kmax).

The stopping condition for the algorithm above is

‖∆v(k)‖ ≤ tol .

Page 16: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Consider the 200 by 200 matrix A bwm200.mtxfrom the matrix market library. It is the discretisedJacobian of the Brusselator wave model for achemical reaction. The resulting eigenvalue problemwith B = I was also studied in Parlett & Saad andwe are interested in finding the rightmost eigenvalueof A which is closest to the imaginary axis and itscorresponding eigenvector.

Page 17: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

α(0) = 0.0, β(0) = 2.5 in line with Parlett & Saad andtook z(0)1 = 1

2‖1‖ and z(0)2 = 1√

32‖1‖ , where 1 is the

vector of all ones.

Page 18: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

k α(k) β(k) ‖w(k+1) ‖λ(k+1) ‖∆v(k)‖ ‖F(v(k))‖−w(k)‖ −λ(k)‖

0 0.00 2.50 3.8e+00 7.8e-01 3.9e+00 3.6e+011 2.34e-1 1.75 1.8e+00 2.2e-01 1.8e+00 7.8e+002 1.18e-1 1.94 8.1e-01 1.4e-01 8.2e-01 1.7e+003 4.47e-2 2.06 2.5e-01 7.0e-02 2.6e-01 3.4e-014 8.82e-3 2.12 3.1e-02 1.7e-02 3.5e-02 3.7e-025 2.48e-4 2.13 4.8e-04 5.2e-04 7.1e-04 7.1e-046 1.80e-5 2.13 1.2e-07 2.5e-07 2.8e-07 2.8e-077 1.81e-5 2.13 2.1e-14 2.9e-14 3.6e-14 6.0e-14

Page 19: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Newton’s method in complex arithmetic

A,v(0) = [z(0)1 , z(0)2 , α(0), β(0)]T , kmax& tol.For k = 0,1,2, . . . , until convergenceCompute the LU factorisation of[

A− λ(k)I −z(k)

−(z(k))H 0

].

d(k) = −[(A− λ(k)I)z(k)

−12z(k)

Hz(k) + 1

2

].

Solve Ly(k) = d(k) for y(k).Solve U∆v(k) = y(k) for ∆v(k).Update v(k+1) = v(k) + ∆v(k).

Page 20: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Newton’s method in Complex Arithmetic

k α(k) + iβ(k) ‖z(k+1) |λ(k+1) ‖∆v(k)‖ ‖F(v(k))‖−z(k)‖ −λ(k)|

0 0.00+2.50i 3.8e+00 7.8e-01 3.9e+00 3.6e+011 2.34e-1+1.75i 1.8e+00 2.2e-01 1.8e+00 7.8e+002 1.18e-1+1.94i 8.1e-01 1.4e-01 8.2e-01 1.7e+003 4.47e-2+2.06i 2.5e-01 7.0e-02 2.6e-01 3.4e-014 8.82e-3+2.12i 3.1e-02 1.7e-02 3.5e-02 3.7e-025 2.48e-4+2.13i 4.8e-04 5.2e-04 7.1e-04 7.1e-046 1.80e-5+2.13i 1.2e-07 2.5e-07 2.8e-07 2.8e-077 1.81e-5+2.13i 1.1e-14 3.7e-14 3.8e-14 6.3e-14

Page 21: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Quadratic convergence.No need to worry about the choice of c.Strange: If we neglect differentiability, we stillobtained quadratic convergence for B = I.

Page 22: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

Acknowledgements

Everyone presentUniversity of Bath for Funding during my Ph. D.

Page 23: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

G. W. Stewart.Matrix Algorithms, volume II: Eigensystems.SIAM, 2001.

E. Kreyszig.Advanced Engineering Mathematics.John Wiley & Sons, Inc., New York, eighthedition, 1999.

A. Ruhe.Algorithms for the Nonlinear EigenvalueProblem.SIAM J. Matrix Anal. Appl., 10(4):674–689,1973.

B. N. Parlett and Y. Saad.Complex Shift and Invert Strategies for RealMatrices.Lin. Alg. Appl., pages 575–595, 1987.

Page 24: Numerical computation of the Complex Eigenpair of a Large …sanum.github.io/2016/slides/Akinola.pdf · Let A 2Rn n be a large, sparse, nonsymmetric matrix. B 2R n, Symmetric Positive

K. Meerbergen, and D. Roose.Matrix Transformations for Computing RightmostEigenvalues of Large Sparse Non-SymmetricEigenvalue Problems.IMA Journal of Numerical Analysis, 16:297–346,1996.

F. Tisseur.Newton’s Method in Floating Point Arithmeticand Iterative Refinement of GeneralizedEigenvalue Problems.SIAM J. Matrix Anal. Appl., 22:1038–1057, 2001.

P. Deuflhard.Newton Methods for Nonlinear Problems,chapter 4, pages 174–175. Springer, 2004.

B. Boisvert, R. Pozo, K. Remington, B. Miller,and R. Lipman. Matrix Market.http://math.nist.gov/MatrixMarket/.

R. O. Akinola and A. Spence.Two-norm normalization for the matrix pencil:Inverse iteration with a complex shift.International Journal of Innovation in Scienceand Mathematics, 2(5):435–439, 2014.

S. Boyd.Lecture 8: Least Norm Solutions ofUnder-determined Equations, EE263 Autumn2008-09.

R. O. Akinola.Theoretical expression for the nullvector of thejacobian: Inverse iteration with a complex shift.International Journal of Innovation in Scienceand Mathematics, 2(4):367–371, 2014.

M. A. Freitag, and A. Spence.The Calculation of the Distance to Instability bythe Computation of a Jordan Block.Submitted: Linear Algebra and its Application,August 2009.

R. O. Akinola and A. Spence.Numerical Computation of the ComplexEigenvalues of a Matrix by solving a SquareSystem of Equations. Submitted.