|
本帖最后由 hbghlyj 于 2024-10-19 14:30 编辑 Modulo Reduction
It is often a good idea to look at the coefficients of the polynomial from a number theoretical standpoint. The general principle is that any polynomial equation can be reduced mod $m$ to obtain another polynomial equation whose coefficients are the residue classes mod $m$.
Many criterions exist for testing whether a polynomial is irreducible. Unfortunately, none are powerful enough to be universal. One of the most well-known criteria is Eisenstein's criterion.
Theorem 2 (Eisenstein). Let $f(x)=a_{n} x^{n}+a_{n-1} x^{n-1}+\cdots+a_{1} x+a_{0}$ be a polynomial with integer coefficients such that $p \mid a_{i}$ for $0≤i≤n-1, p \nmid a_{n}$ and $p^{2} \nmid a_{0}$. Then $f(x)$ is irreducible.
Proof. Suppose that $f=g h$, where $g$ and $h$ are nonconstant integer polynomials. Consider the reduction $\bmod p$ (i.e., apply the ring homomorphism $ℤ[x] \rightarrow \mathbb{F}_{p}[x]$ ), and let $\bar{f}, \bar{g}, \bar{h}$ denote the residues of $f, g, h$ (i.e. the coefficients are residues $\bmod p)$. We have $\bar{f}(x)=a_{0} x^{n}$. Since $\mathbb{F}_{p}[x]$ is a unique factorization domain, we see that the only possibilities for $\bar{g}$ and $\bar{h}$ are $c x^{k}$ for some integers $c$ and $k \geq 1$. Then, the constant terms of $g$ and $h$ are both divisible by $p$, so $p^{2} \mid a_{0}$. Contradiction.□
The most typical example for the application of Eisenstein's criterion is to show that the cyclotomic polynomial $\Phi_{p}(x)$ is irreducible for prime $p$ :
Problem 1. Let $p$ be a prime number. Show that $f(x)=x^{p-1}+x^{p-2}+\cdots+x+1$ is irreducible.
Solution. The polynomial $f(x)$ is irreducible if and only if $f(x+1)$ is irreducible. We have
$$
f(x+1)=\frac{(x+1)^{p}-1}{(x+1)-1}=x^{p-1}+\left(\begin{array}{l}
p \\
1
\end{array}\right) x^{p-2}+\left(\begin{array}{l}
p \\
2
\end{array}\right) x^{p-3}+\cdots+\left(\begin{array}{c}
p \\
p-2
\end{array}\right) x+p
$$
Note that $f(x+1)$ fails the Eisenstein criterion for the prime $p$. Therefore $f(x)$ is irreducible.□
Note that the proof of Eisenstein's criterion extends to other rings with similar properties. For instance, to show that $x^{4}+5 x+5$ is irreducible over the Gaussian integers $ℤ[i ]$, we can simply apply Eisenstein with the Gaussian prime $2+i$.
The proof of Eisenstein's Criterion can be slightly generalized to the following. The proof is more or less the same, and so it's left as exercise.
Theorem 3 (Extended Eisenstein). Let $f(x)=a_{n} x^{n}+a_{n-1} x^{n-1}+\cdots+a_{1} x+a_{0}$ be a polynomial with integer coefficients such that $p \mid a_{i}$ for $0≤i<k, p \nmid a_{k}$ and $p^{2} \nmid a_{0}$. Then $f(x)$ has an irreducible factor of degree greater than $k$.
We give one more result that relates to looking at the modulo reduction of polynomials, known as Hensel's lemma.
Theorem 4 (Hensel). Let $a_{0}, a_{1}, \ldots, a_{k}$ be integers, and let $P(x)=a_{n} x^{k}+\cdots a_{1} x+a_{0}$, and let $P'(x)$ denote the derivative of $P(x)$. Suppose that $x_{1}$ is an integer such that $P\left(x_{1}\right) \equiv 0\pmod p$ and $P'\left(x_{1}\right) \not \equiv 0\pmod p$. Then, for any positive integer $k$, there exists an unique residue $x\pmod{p^k}$, such that $P\left(x_{k}\right) \equiv 0\pmod{p^k}$ and $x \equiv x_{1}\pmod p$.
The proof of Hensel's lemma closely mimics Newton's method of finding roots. We work up the powers of $p$, and find the a zero of $P(x) \bmod p^{k}$ for $k=2,3, \ldots$ The details of the proof are omitted here.
Root Hunting
When working with integer polynomials, it is often not enough to stay in $ℤ$. We have to think outside the box and move our scope to the complex numbers. A lot can be a said about a polynomial if we know something about its complex zeros. Many irreducibility problems hinge on placing bounds on the zeros of the polynomial in the complex plane. We begin with a familiar example.
Problem 2. Let $f(x)=a_{n} x^{n}+a_{n-1} x^{n}+\cdots+a_{1} x+a_{0}$ be a polynomial with integer coefficients, such that $\left|a_{0}\right|$ is prime and
$$
\left|a_{0}\right|>\left|a_{1}\right|+\left|a_{2}\right|+\cdots+\left|a_{n}\right| .
$$
Show that $f(x)$ is irreducible.
Solution. Let $\alpha$ be any complex zero of $f$. Suppose that $|\alpha|≤1$, then
$$
\left|a_{0}\right|=\left|a_{1} \alpha+\cdots+a_{n} \alpha^{n}\right| \leq\left|a_{1}\right|+\cdots+\left|a_{n}\right|
$$
a contradiction. Therefore, all the zeros of $f$ satisfies $|\alpha|>1$.
Now, suppose that $f(x)=g(x) h(x)$, where $g$ and $g$ are nonconstant integer polynomials. Then $a_{0}=$ $f(0)=g(0) h(0)$. Since $\left|a_{0}\right|$ is prime, one of $|g(0)|,|h(0)|$ equals 1. Say $|g(0)|=1$, and let $b$ be the leading coefficient of $g$. If $\alpha_{1}, \ldots, \alpha_{k}$ are the roots of $g$, then $\left|\alpha_{1} \alpha_{2} \cdots \alpha_{k}\right|=1 /|b|≤1$. However, $\alpha_{1}, \ldots, \alpha_{k}$ are also zeros of $f$, and so each has an magnitude greater than 1 . Contradiction. Therefore, $f$ is irreducible.□
Next, we present a Perron's criterion, which has a similar statement but a much more difficult proof compared with the previous result.
Theorem 5 (Perron). Let $P(x)=x^{n}+a_{n-1} x^{n-1}+\cdots+a_{1} x+a_{0}$ be a polynomial with $a_{0} \neq 0$ and
$$
\left|a_{n-1}\right|>1+\left|a_{n-2}\right|+\cdots+\left|a_{1}\right|+\left|a_{0}\right|
$$
Then $P(x)$ is irreducible.
Again, the idea is to put bounds on the modulus of the roots of $f$. The key lies in the following lemma.
Lemma 1. Let $P(x)=x^{n}+a_{n-1} x^{n-1}+\cdots+a_{1} x+a_{0}$ be a polynomial with
$$
\left|a_{n-1}\right|>1+\left|a_{n-2}\right|+\cdots+\left|a_{1}\right|+\left|a_{0}\right| .
$$
Then exactly one zero of $P$ satisfies $|z|>1$, and the other $n-1$ zeros of $P$ satisfy $|z|<1$.
Let us see how we can prove Perron's criterion if we have this lemma. Suppose that $P(x)=f(x) g(x)$, where $f$ and $g$ are integer polynomials. Since $P$ has only one zero with modulus not less than 1 , one of the polynomials $f, g$, has all its zeros strictly inside the unit circle. Suppose that $z_{1}, \ldots, z_{k}$ are the zeros of $f$, and $\left|z_{1}\right|, \ldots,\left|z_{k}\right|<1$. Note that $f(0)$ is a nonzero integer, and $|f(0)|=\left|z_{1} \cdots z_{k}\right|<1$, contradiction. Therefore, $f$ is irreducible.
Now, let us prove Lemma 1. We offer two proofs. The first proof is an elementary proof that uses only the triangle inequality. The second proof invokes theorems from complex analysis, but it is much more intuitive and instructive.
First proof of the Lemma 1. (due to Laurentiu Panaitopol) Let us suppose wlog that $a_{0} \neq 0$ since we can remove any factors of the form $x^{k}$. Let's first prove that there is no root $\alpha$ of $P(x)$ with $|\alpha|=1$. Suppose otherwise, then we have that
$$
-a_{n-1} \alpha^{n-1}=\alpha^{n}+a_{n-2} \alpha^{n-2}+\cdots+a_{1} \alpha+a_{0}
$$
thus
$$
\begin{aligned}
\left|a_{n-1}\right|=\left|a_{n-1} \alpha^{n-1}\right| &=\left|\alpha^{n}+a_{n-2} \alpha^{n-2}+\cdots+a_{1} \alpha+a_{0}\right| \\
& \leq\left|\alpha^{n}\right|+\left|a_{n-2} \alpha^{n-2}\right|+\cdots+\left|a_{1} \alpha\right|+\left|a_{0}\right| \\
&=1+\left|a_{n-2}\right|+\cdots+\left|a_{1}\right|+\left|a_{0}\right|
\end{aligned}
$$
This contradicts the given inequality. Therefore, no zero of $f(x)$ lies on the unit circle.
Let's denote with $\alpha_{1}, \alpha_{2}, \ldots, \alpha_{n}$ be the zeros of $P$. Since $\left|\alpha_{1} \alpha_{2} \cdots \alpha_{n}\right|=a_{0}$, it follows that at least one of the roots is larger than 1 in absolute value. Suppose that $\left|\alpha_{1}\right|>1$ and let
$$
Q(x)=x^{n-1}+b_{n-2} x^{n-2}+\cdots+b_{1} x+b_{0}
$$
be the polynomial with roots $\alpha_{2}, \alpha_{3}, \ldots, \alpha_{n}$. Then,
$$
P(x)=\left(x-\alpha_{1}\right) Q(x)=x^{n}+\left(b_{n-2}-\alpha_{1}\right) x^{n-1}+\left(b_{n-3}-b_{n-2} \alpha_{1}\right) x^{n-2}+\cdots+\left(b_{0}-b_{1} \alpha_{1}\right) x-b_{0} \alpha_{1}
$$
It follows that $b_{n-1}=1, a_{0}=-b_{0} \alpha_{1}$, and $a_{k}=b_{k-1}-b_{k} \alpha_{1}$ for all $1≤k≤n-1$. Then, using the given inequality, we have
$$
\begin{aligned}
\left|b_{n-2}-\alpha_{1}\right|=\left|a_{n-1}\right| &>1+\left|a_{n-2}\right|+\cdots+\left|a_{1}\right|+\left|a_{0}\right| \\
&=1+\left|b_{n-3}-b_{n-2} \alpha_{1}\right|+\cdots+\left|b_{0} \alpha_{1}\right| \\
& \geq 1+\left|b_{n-2}\right|\left|\alpha_{1}\right|-\left|b_{n-3}\right|+\left|b_{n-3}\right|\left|\alpha_{1}\right|-\left|b_{n-4}\right|+\cdots+\left|b_{1}\right|\left|x_{1}\right|-\left|b_{0}\right|+\left|b_{0}\right|\left|x_{1}\right| \\
&=1+\left|b_{n-2}\right|+\left(\left|\alpha_{1}\right|-1\right)\left(\left|b_{n-2}\right|+\left|b_{n-3}\right|+\cdots+\left|b_{1}\right|+\left|b_{0}\right|\right)
\end{aligned}
$$
On the other hand, $\left|b_{n-2}-\alpha_{1}\right| \leq\left|b_{n-2}\right|+\left|\alpha_{1}\right|$, so
$$
\left|b_{n-2}\right|+\left|\alpha_{1}\right|>1+\left|b_{n-2}\right|+\left(\left|\alpha_{1}\right|-1\right)\left(\left|b_{n-2}\right|+\left|b_{n-3}\right|+\cdots+\left|b_{1}\right|+\left|b_{0}\right|\right)
$$
and therefore
$$
\left|b_{n-2}\right|+\left|b_{n-3}\right|+\cdots+\left|b_{1}\right|+\left|b_{0}\right|<1
$$
Then, for any complex number $\alpha$ with $|\alpha| \geq 1$, we have
$$
\begin{aligned}
|Q(\alpha)| &=\left|\alpha^{n-1}+b_{n-2} \alpha^{n-2}+b_{n-3} \alpha^{n-3}+\cdots+b_{1} \alpha+b_{0}\right| \\
& \geq\left|\alpha^{n-1}\right|-\left|b_{n-2} \alpha^{n-2}\right|-\left|b_{n-3} \alpha^{n-3}\right|-\cdots-\left|b_{1} \alpha\right|-\left|b_{0}\right| \\
& \geq|\alpha|^{n-1}-|\alpha|^{n-1}\left(\left|b_{n-2}\right|+\left|b_{n-3}\right|+\cdots+\left|b_{1}\right|+\left|b_{0}\right|\right) \\
&=|\alpha|^{n-1}\left(1-\left|b_{n-2}\right|-\left|b_{n-3}\right|-\cdots-\left|b_{1}\right|-\left|b_{0}\right|\right) \\
&>0
\end{aligned}
$$
And so $\alpha$ cannot be a root. It follows that all the zeros of $Q$ lie strictly inside the unit circle. This completes the proof of the lemma.
In the polynomial $P$, the second term $x^{n-1}$ is "dominating," in the sense that the absolute value of its coefficient is greater than the sum of the absolute values of all the other coefficients. In the above proof, we managed to construct a new polynomial $Q$, whose leading term is dominating. While exactly one zero of $P$ is outside the unit circle, none of the zeros of $Q$ is outside the unit circle. This observation generalizes to the following result.
Proposition 6. Let $P(z)=a_{n} z^{n}+a_{n-1} z^{n-1}+\cdots+a_{1} z+a_{0}$ be a polynomial with complex coefficients, and such that
$$
\left|a_{k}\right|>\left|a_{0}\right|+\left|a_{1}\right|+\cdots+\left|a_{k-1}\right|+\left|a_{k+1}\right|+\cdots+\left|a_{n}\right|
$$
for some $0≤k≤n$. Then exactly $k$ zeros of $P$ lie strictly inside the unit circle, and the other $n-k$ zeros of $P$ lie strictly outside the unit circle.
This is indeed true. The easiest way to prove this result is to invoke a well-known theorem in complex analysis, known as Rouché's theorem.
Theorem 7 (Rouché). Let $f$ and $g$ be analytic functions on and inside a simple closed curve $\mathcal{C}$. Suppose that $|f(z)|>|g(z)|$ for all points $z$ on $\mathcal{C}$. Then $f$ and $f+g$ have the same number of zeros (counting multiplicities) interior to $\mathcal{C}$.
The proof of Rouché's theorem uses the argument principle. It can be found in any standard complex analysis textbook.
In practice, for polynomials, Rouché's theorem is generally applied to some circle, and is useful when one term is very big compared to the other terms.
Proposition 6 becomes very easy to prove with the aid of Rouché's theorem. Indeed, let us apply Rouché's theorem to the functions $a_{k} z^{k}$ and $P(z)-a_{k} z^{k}$ with the curve being the unit circle. The given inequality implies that $\left|a_{k} z^{k}\right|>\left|P(z)-a_{k} z^{k}\right|$ for all $|z|=1$. It follows that $P$ has the same number of zeros as $a_{k} z^{k}$ inside the unit circle. It follows that $P$ has exactly $k$ zeros inside the unit circle. Also, it is not hard to show that $P$ has no zeros on the unit circle (c.f. first proof of Lemma 1). Thus we have proved Proposition 6 .
Second proof of Lemma 1. Apply Proposition 6 to $k=n-1$.
While we're at it, let's look at couple of neat applications of Rouché's theorem, just for fun. These are not integer polynomial problems, but they contain useful ideas.
Problem 3. (Romania ??) Let $f \in \mathbb{C}[x]$ be a monic polynomial. Prove that we can find a $z \in \mathbb{C}$ such that $|z|=1$ and $|f(z)| \geq 1$.
Solution. Let $\operatorname{deg} P=n$. Suppose that $|f(z)|<1$ for all $z$ on the unit circle. Then $|f(z)|<\left|z^{n}\right|$ for all $z$ on the unit circle. So, by Rouché's theorem, $f(z)-z^{n}$ has $n$ roots inside the unit circle, which is impossible, since $f(z)-z^{n}$ has degree $n-1$.
The Fundamental Theorem of Algebra is also an easy consequence of Rouché's theorem.
Theorem 8 (Fundamental Theorem of Algebra). Any polynomial $P(x) \in \mathbb{C}[x]$ of degree $n$ has exactly $n$ complex zeros.
Proof. Let $P(x)=a_{n} x^{n}+\cdots+a_{1} x+a_{0}$. For a sufficiently large real number $R$, we have
$$
\left|a_{n}\right| R^{n}>\left|a_{n-1}\right| R^{n-1}+\cdots+\left|a_{1}\right| R+a_{0} .
$$
Apply Rouché's theorem to the functions $a_{n} x^{n}$ and $P(x)-a_{n} x^{n}$ on the circle $|z|=R$, we find that $P(x)$ has exactly $n$ zeros inside the circle. Also, since we may choose $R$ arbitrarily large, so there are no additional zeros.
Note that the above proof also gives a bound (although rather weak) for the zeros of a polynomial. This bound is attributed to Cauchy.
Finally, the following result is a slightly stronger version of Rouché's theorem.
Theorem 9 (Extended Rouché). Let $f$ and $g$ be analytic functions on and inside a simple closed curve $\mathcal{C}$. Suppose that
$$
|f(z)+g(z)|<|f(z)|+|g(z)|
$$
for all points $z$ on $\mathcal{C}$. Then $f$ and $g$ have the same number of zeros (counting multiplicities) interior to $\mathcal{C}$.
There are many ways of bounding polynomial zeros on the complex plane. The following result is worth mentioning, as it has proven useful quite a few times.
Proposition 10. Let $P(x)=a_{0}+a_{1} x+\cdots+a_{n} x^{n}$, where $0<a_{0}≤a_{1}≤\cdots≤a_{n}$ are real numbers, then any complex zero of the polynomial satisfies $|z|≤1$.
Proof. If $|z|>1$, then, since $z$ is a zero of $(1-x) P(x)$, we get
$$
a_{0}+\left(a_{1}-a_{0}\right) z+\cdots+\left(a_{n}-a_{n-1}\right) z^{n}-a_{n} z^{n}=0 .
$$
Thus,
$$
\begin{aligned}
\left|a_{n} z^{n}\right| &=\left|a_{0}+\left(a_{1}-a_{0}\right) z+\cdots+\left(a_{n}-a_{n-1}\right) z^{n}\right| \\
&≤a_{0}+\left(a_{1}-a_{0}\right)|z|+\cdots+\left(a_{n}-a_{n-1}\right)\left|z^{n}\right| \\
&<a_{0}|z|^{n}+\left(a_{1}-a_{0}\right)|z|^{n}+\cdots+\left(a_{n}-a_{n-1}\right)|z|^{n} \\
&=a_{0}|z|^{n}-a_{0}|z|^{n}+a_{1}|z|^{n}-a_{1}|z|^{n}+\cdots+a_{n}|z|^{n} \\
&=\left|a_{n} z^{n}\right|
\end{aligned}
$$
contradiction. Therefore, $|z| ≤ 1$.□
It follows as a simple corollary that for any polynomial with positive real coefficients, $P(x)=a_{0}+a_{1} x+$ $\cdots+a_{n} x^{n}$, all its zeros lie in the annulus
$$
\min _{1≤k≤n} \frac{a_{k-1}}{a_{k}} \leq|z|≤\max _{1≤k≤n} \frac{a_{k-1}}{a_{k}}
$$
Finally, we present one more irreducibility criterion, known as Cohn's criterion. Essentially, it says that if $f(x)$ has nonnegative integer coefficients, and $f(n)$ is prime for some $n$ greater than all the coefficients, then $f$ is irreducible.
Theorem 11 (Cohn's Criterion). Let $p$ be a prime number, and $b \geq 2$ an integer. Suppose that $\overline{p_{n} p_{n-1} \cdots p_{1} p_{0}}$ is the base- $b$ representation of $p$, with $0≤p_{i}<b$ for each $i$ and $p_{n} \neq 0$, then the polynomial
$$
f(x)=p_{n} x^{n}+p_{n-1} x^{n}+\cdots+p_{1} x+p_{0}
$$
is irreducible.
The following proof is due to M. Ram Murty
M. Ram Murty, Prime Numbers and Irreducible Polynomials, Amer. Math. Monthly. 10.pdf
(86.55 KB, 下载次数: 0)
As before, we begin with a lemma bounding the complex zeros of the polynomial.
Lemma 2. Let $f(x)=a_{n} x^{n}+a_{n-1} x^{n-1}+\cdots+a_{1} x+a_{0}$ belong to $ℤ[x]$. Suppose that $a_{n} \geq 1, a_{n-1} \geq 0$, and $\left|a_{i}\right|≤H$ for $i=0,1, \ldots, n-2$, where $H$ is some positive constant. Then any complex zero $\alpha$ of $f(x)$ either has nonpositive real part, or satisfies
$$
|\alpha|<\frac{1+\sqrt{1+4 H}}{2}
$$
Proof. If $|z|>1$ and $\operatorname{Re} z>0$, we observe that
$$
\begin{aligned}
\left|\frac{f(z)}{z^{n}}\right| & \geq\left|a_{n}+\frac{a_{n-1}}{z}\right|-H\left(\frac{1}{|z|^{2}}+\cdots \frac{1}{|z|^{n}}\right) \\
&>\operatorname{Re}\left(a_{n}+\frac{a_{n-1}}{z}\right)-\frac{H}{|z|^{2}-|z|} \\
& \geq 1-\frac{H}{|z|^{2}-|z|}=\frac{|z|^{2}-|z|-H}{|z|^{2}-|z|} \geq 0
\end{aligned}
$$
whenever
$$
|z| \geq \frac{1+\sqrt{1+4 H}}{2}
$$
It follows that $\alpha$ cannot be a zero of $f$ if $|\alpha| \geq \frac{1+\sqrt{1+4 H}}{2}$ and $\operatorname{Re} \alpha>0$.
To prove Theorem 11 for the case $b \geq 3$, we notice that Lemma 2 implies if $\alpha$ is a zero of $f(x)$, then $|b-\alpha|>1$. Suppose that $f(x)=g(x) h(x)$, where $g$ and $h$ are nonconstant integer polynomials. Since $f(b)$ is prime, one of $|g(b)|,|h(b)|$ is 1 . Say $|g(b)|=1$, and the zeros of $g$ are $\alpha_{1}, \ldots, \alpha_{k}$. We have $|g(b)|=\left|b-\alpha_{1}\right| \cdots\left|b-\alpha_{k}\right|>1$, contradiction. Therefore, $f$ is irreducible.
The $b=2$ case is special, and requires more analysis.
Lemma 3. Let $f(x)=x^{n}+a_{n-1} x^{n-2}+\cdots+a_{1} x+a_{0}$ with $a_{i} \in\{0,1\}$ for each $i$. Then all the zeros of $f$ lie in the half plane $\operatorname{Re} z<\frac{3}{2}$.
Proof. The cases $n=1$ and 2 can be verified by hand. Assume that $n \geq 3$. Then, for $z \neq 0$, we have
$$
\left|\frac{f(z)}{z^{n}}\right| \geq\left|1+\frac{a_{n-1}}{z}+\frac{a_{n-2}}{z^{2}}\right|-\left(\frac{1}{|z|^{3}}+\cdots+\frac{1}{|z|^{n}}\right)>\left|1+\frac{a_{n-1}}{z}+\frac{a_{n-2}}{z^{2}}\right|-\frac{1}{|z|^{2}(|z|-1)}
$$
If $z$ satisfies $|\arg z|≤\pi / 4$, then we have $\operatorname{Re}\left(1 / z^{2}\right) \geq 0$, and we get
$$
\left|\frac{f(z)}{z^{n}}\right|>1-\frac{1}{|z|^{2}(|z|-1)} .
$$
If $|z| \geq \frac{3}{2}$, then $|z|^{2}(|z|-1) \geq\left(\frac{3}{2}\right)^{2}\left(\frac{3}{2}-1\right)=\frac{9}{8}>1$, and so $f(z) \neq 0$. On the other hand, if $z$ is a zero of $f$ with $|\arg z|>\pi / 4$, and suppose that $\operatorname{Re} z>0$, then from Lemma 2 we have $|z|<\frac{1+\sqrt{5}}{2}$, and thus $\operatorname{Re} z<\frac{1+\sqrt{5}}{2 \sqrt{2}}<\frac{3}{2}$. It follows that all zeros of $f$ lie in the half-plane $\operatorname{Re} z<\frac{3}{2}$.
To finish off the proof, suppose that $f(x)=g(x) h(x)$, where $g$ and $h$ are integer polynomials. Since $f(2)$ is prime, one of $|g(2)|,|h(2)|$ is 1. Say $|g(2)|=1$. By Lemma 3, all the zeros of $f$ lie in the half plane $\operatorname{Re}z<\frac{3}{2}$, which means that they satisfy $|z-2|>|z-1|$. Thus, if $\alpha_{1}, \ldots, \alpha_{k}$ are the zeros of $g$, we have $|g(2)|=\left|2-\alpha_{1}\right| \cdots\left|2-\alpha_{k}\right|>\left|1-\alpha_{1}\right| \cdots\left|1-\alpha_{k}\right|=|g(1)| \geq 1$. So $|g(2)|>1$, contradiction. |
|