Zulip Chat Archive

Stream: maths

Topic: an optimization problem


Alex Zhang (Oct 20 2021 at 18:02):

Given an arbitrary square matrix with the row sum of each row fixed. Could anyone explain or hint how to rigorous establish that a matrix with pairwisely perpendicular rows (properly ordered) is an optimal solution to the determinant optimization problem?

Yaël Dillies (Oct 20 2021 at 18:36):

It might be related to the Birkhoff-Von Neumann problem? If the determinant is convex in any useful way (not sure convexity even makes sense), then you know it's maximized on doubly stochastic matrices (which what you asked for, unless you're allowed negative coefficients?) by an extreme point, which is a permutation matrix thanks to Birkhoff-Von Neumann.

Yaël Dillies (Oct 20 2021 at 18:37):

I just made all of that up so don't take my word for it.

David Wärn (Oct 20 2021 at 19:09):

I think what you really want is to fix the sum-of-squares in each row? For positive entries you can relate this to the sum via ixi2(xi)2\sum_i x_i^2 \le (\sum x_i)^2, but otherwise you get very large determinant from for example (10100101)\begin{pmatrix} 1 & 0 \\ -100 & 101 \end{pmatrix}.

David Wärn (Oct 20 2021 at 19:14):

I guess if you have an inner product space VV, there's a well-behaved notion of the kk-volume M(v1vk)M(v_1 \ldots v_k) spanned by kk vectors v1vkv_1 \ldots v_k (say, pick an orthonormal basis of the subspace spanned by them, and look at the absolute value of the determinant of the corresponding k×kk \times k-matrix). For k=dimVk = \dim V this gives you the determinant. And you should be able to prove a bound M(v1vk)iviM(v_1 \ldots v_k) \le \prod_i \lVert v_i \rVert by induction on kk, using a generalization of the "base times height" formula for the area of a parallelogram.

Alex Zhang (Oct 20 2021 at 19:18):

Yes. fix the sum-of-squares

Alex Zhang (Oct 20 2021 at 19:20):

what is the generalization of the "base times height" formula?

David Wärn (Oct 20 2021 at 19:46):

By using Laplace expansion in a suitable basis, you should be able to show that M(v1vk+1)=M(v1vk)vk+1uM(v_1 \ldots v_{k+1}) = M(v_1 \ldots v_k) \lVert v_{k+1} - u \rVert, where uu is the projection of vk+1v_{k+1} onto the subspace spanned by v1vkv_1 \ldots v_k

David Wärn (Oct 20 2021 at 19:47):

Btw I have no idea what would be the best way to formalize this result in mathlib

Alex Zhang (Oct 20 2021 at 20:14):

This seems like a reasonable way to formally prove the result, but I feel it can be tedious to encode it.

Kyle Miller (Oct 20 2021 at 20:37):

This seems like a job for Lagrange multipliers and Jacobi's formula. A sketch:

First, consider the submanifold of k×kk\times k matrices where row ii has length cic_i, with c1,,ck>0c_1,\dots,c_k>0. This submanifold is a level set of A(v1,,vk)A\mapsto (\lVert v_1\rVert,\dots,\lVert v_k\rVert) for the codomain point (c1,,ck)(c_1,\dots,c_k), and let AA denote a matrix in this submanifold. Let AiA_i denote the matrix AA, but setting all but row ii to 00. The matrices A1,,AkA_1,\dots,A_k span the subspace of the tangent bundle that are orthogonal to the submanifold at AA.

One version of Jacobi's formula is that det(A)/Aij=adj(A)ji\partial\det(A)/\partial{A_{ij}} = \operatorname{adj}(A)_{ji}, where AijA_{ij} is entry (i,j)(i,j) of AA. A critical point of det\det when restricted to the submanifold corresponds to a matrix AA where the matrix (det(A)/Aij)ij(\partial\det(A)/\partial{A_{ij}})_{ij} lies in the subspace spanned by A1,,AkA_1,\dots,A_k, thus we can say each column of adj(A)\operatorname{adj}(A) is a scalar multiple of the corresponding row of AA.

Assuming det(A)0\det(A)\neq 0, then AA is invertible, so adj(A)=det(A)A1\operatorname{adj}(A)=\det(A)A^{-1}. Since AA1=IAA^{-1}=I, putting this all together the rows of AA are pairwise perpendicular. We can ignore det(A)=0\det(A)=0 as an optimum since the diagonal matrix with c1,,cnc_1,\dots,c_n on the diagonal gives a lower bound for the maximal determinant.

David Wärn (Oct 20 2021 at 21:42):

You can rephrase my argument above to make it more direct: if AA is a square matrix, then you should be able to show that there exists a unitary matrix UU such that AUAU is upper triangular. This has the same (absolute value of) determinant as AA, and the norms of the rows are the same. But now the conclusion is clear, since the determinant is a product of diagonal entries, and the norms are lower bounded by diagonal entries.

Will Sawin (Oct 20 2021 at 21:54):

I think this is called Hadamard's inequality and searching that should give a proof.

Dima Pasechnik (Oct 22 2021 at 10:55):

yes, and in fact a student of mine worked on formalising Hadamard matrices in Liean+mathlib last summer.

Dima Pasechnik (Oct 22 2021 at 11:03):

And this student is @Alex Zhang (hi!) - whom I only recognised from the email :-)

Dima Pasechnik (Oct 22 2021 at 11:07):

Hadamard matrices are ones for which Hadamard inequality turns into equation (one can renormalise the nxn matrix to have its rows and columns to be of squared Euclidean norm n, and entries have norm at most 1 (and thus exactly 1).

Alex Zhang (Oct 23 2021 at 12:25):

Hi, Dima! @Dima Pasechnik


Last updated: Dec 20 2023 at 11:08 UTC