Given the equation \begin{equation}\det(\lambda^2 I+ B \lambda +K )=0\end{equation} where $I,B,K\in \mathbb R^{m \times m}$. $B$ and $K$ are symmetric matrices with no zero eigenvalues and $B>0$. Let $n^+(A)$ and $n^-(A)$ denote the number of eigenvalues of $A$ with positive real parts and negative real parts respectively. Is the number of roots of the above equation with positive real parts equal to $n^-(B)+n^-(K)$ and the number of roots with negative real parts equal to $n^+(B)+n^+(K)$?
My trial was as follows: let $v \in \mathbb{ R^m}$ if $K$ is positive definite then $$\det(\lambda^2 I+ B \lambda +K )=0 \implies \exists v: v^T(\lambda^2 I+ B \lambda +K)v=0 \implies \lambda^2 v^2+ v^TBv \lambda +v^TKv=0.$$ All the coefficients are positive, so real part of $\lambda$ must be negative. The same argument can be used when $K<0$, the remaining case is when $K$ is indefinite.
Edit
As Ben Grossmann showed the system can be seen as the characteristic equation of: $$ J = \pmatrix{0&&I \\ -K && -B}. $$ where $B>0$, $J$ cannot have an eigenvalue with purely imaginary part if it did then $ \exists v: v^H((bi)^2 I+ B (bi) +K)v=0 \implies v^HBvb=0 \iff b=0$
Let $n_0(A)$ denote the number of zero eigenvalues of A.
lemma 1: $n_0(K)=n_0(J)$
we observe that the reduced echelon form of $J$ is: $$ J_{red} = \pmatrix{I&&0\\0 && K}. $$ so $n_0(K)=n_0(J)$.
Let $G(t)=K+t I$ and let $$ J(t)=\pmatrix{0&&I\\-G(t) &&-B} $$ observe that as $t\rightarrow \infty$,$G(t)>0 \implies n_-(J(t))=2m$ and as $t\rightarrow -\infty$ , $G(t)<0 \implies n_-(J(t))=n_+(J(t))=m$. Let the eigenvalues of $J(t)$ be $\{\lambda_i(t)\}$.
As $t$ goes from $-\infty$ to $+\infty$, the eigenvalues of $G(t)$ become zero $m$ times which is when they change signs. By lemma 1, the eigenvalues of $J(t)$ must also become zero $m$ times and those times are exactly when eigenvalues of $G(t)$ are zero. It is not difficult to see that the eigenvalues $J(t)$ are zero exactly when one of the positive eigenvalues change signs to negative, if not then one of the positive eigenvalues of $J(t)$ won't change signs and would remain positive as $t \rightarrow +\infty$ which is a contradiction.
So every time an eigenvalue of $G(t)$ changes signs from negative to positive, an eigenvalue of $J(t)$ will change signs from positive to negative, so we have that $\forall t$ , $n_-(J(t))=m+n_+(G(t))=n_+(B)+n_+(G(t))$, taking $t=0$ yields $n_-(J)=n_+(B)+n_+(K)$ as required.
Is there something wrong with this proof?