Zulip Chat Archive

Stream: maths

Topic: Linear combinations of $$t^ke^{λt}$$


Yury G. Kudryashov (Apr 24 2022 at 20:29):

I'm going to add some facts about functions of the form f(t)=jajtkjeλjtf(t)=\sum_j a_jt^{k_j}e^{λ_jt}. Two use cases I have in mind are

  • solutions of linear differential equations x˙(t)=Ax(t)+f(t)\dot x(t)=Ax(t)+f(t);
  • they naturally appear as partial sums of asymptotic series expansion of the correspondence map of a hyperbolic saddle point.

I have a few questions:

  1. How should I call them? I saw the name "quasi polynomials" in some sources (mostly in Russian) but wiki disagrees.
  2. How general should be the definition? I know about applications in these cases:

    • all aja_j, λjλ_j, and tt are numbers (real or a complex);
    • aja_j is a matrix, λjλ_j and tt are real or complex numbers;
    • aja_j and tt are numbers, λjλ_j is a matrix (actually, it is λjAλ_jA).

Kevin Buzzard (Apr 24 2022 at 21:08):

Is this finite sums you're talking about?

Yury G. Kudryashov (Apr 24 2022 at 21:16):

Yes.

Yury G. Kudryashov (Apr 24 2022 at 21:39):

Let me elaborate on applications.

Linear ODEs

If AA is a matrix with eigenvalues λjλ_j with multiplicities rjr_j, then x(t)=eAtx(0)x(t)=e^{At}x(0). If we rewrite this in coordinates, xk(t)=jPk,j(t)eλjtx_k(t)=\sum_j P_{k,j}(t)e^{λ_jt}, where Pk,jP_{k,j} is a polynomial of degree at most rj1r_j-1.

Dulac series

Let Δ ⁣:(R+,0)(R+,0)Δ\colon (\mathbb R_+, 0) → (\mathbb R_+, 0) be the correspondence map of an analytic hyperbolic saddle and F(t)=lnΔ(et)F(t)=-\ln Δ(e^{-t}), F ⁣:(R+,)(R+,)F\colon (\mathbb R_+, \infty)\to(\mathbb R_+, \infty), be the same map written in the logarithmic chart. Then for each Λ>0Λ>0 we have

F(t)=at+b+j=1N(Λ)Pj(t)eλjt+o(eΛt)F(t)=at+b+\sum_{j=1}^{N(Λ)} P_j(t)e^{-λ_jt}+o(e^{-Λt})

as tt\to\infty, where 0<λjΛ0<λ_j\le Λ and PjP_j are polynomials. The functions in the RHS can be glued into an asymptotic series

at+b+j=1Pj(t)eλjt.at+b+\sum_{j=1}^∞ P_j(t)e^{-λ_jt}.

This series may diverge but it is an asymptotic series for FF.

Moreover, the same asymptotic expansion holds true in the image ΩC\Omega_C of the complex right half-plane under the map zz+C1+zz\mapsto z+C\sqrt{1+z} for sufficiently large positive CC. The latter fact together with a special version of the Phragmen-Lindelöf principle implies that the Poincaré map of a hyperbolic polycycle is either the identity map, or has an isolated fixed point at zero (Ilyashenko, about 1990).

Eric Wieser (Apr 24 2022 at 21:40):

Note I've made a bunch of progress on matrix exponentials specifically with (the first half of) that first example in mind

Yury G. Kudryashov (Apr 24 2022 at 21:41):

My main goal is the second application but IMHO we should have a definition that works in both cases.

Yury G. Kudryashov (Apr 24 2022 at 21:47):

For the second application, I want to have theorems like

j=1NPj(t)eλjt=a1td1eλ1t+o(td1eλ1t)\sum_{j=1}^{N}P_j(t)e^{-λ_jt} = a_1t^{d_1}e^{-λ_1t}+o(t^{d_1}e^{-λ_1t})

as tt\to\infty, where a1td1a_1t^{d_1} is the leading term of P1(t)P_1(t) and λ1>λ2>λ_1>λ_2>…

Yury G. Kudryashov (Apr 24 2022 at 21:49):

Actually, I need this as re t → ∞ or abs t → ∞ while tΩCt∈\Omega_C.

Yury G. Kudryashov (May 07 2022 at 04:25):

#13178 is ready for review; this kind of quasi polynomials is the next item on my Lean TODO list. Any ideas about the name and typeclass assumptions?


Last updated: Dec 20 2023 at 11:08 UTC