Polynomial $x^p-x+a$ is Irreducible and Separable Over a Finite Field

Problems and Solutions in Field Theory in Abstract Algebra

Problem 229

Let $p\in \Z$ be a prime number and let $\F_p$ be the field of $p$ elements.
For any nonzero element $a\in \F_p$, prove that the polynomial
\[f(x)=x^p-x+a\] is irreducible and separable over $F_p$.

(Dummit and Foote “Abstract Algebra” Section 13.5 Exercise #5 on p.551)

 
LoadingAdd to solve later

Sponsored Links

Proof.

Separability

The separability can be checked by noting that the derivative of $f(x)$ is
\[f'(x)=px^{p-1}-1=-1\] and is relatively prime to $f(x)$, and thus $f(x)$ is separable.

We give two proofs for the irreducibility of $f(x)=x^p-x+a$. Both proofs use the following lemmas.

Lemma 1

Lemma 1. If $\alpha$ is a root of $f(x)=x^p-x+a$, then $\alpha+j$ is a root of $f(x)$ for any $j\in \F_p$.

Proof of Lemma 1

We have
\begin{align*}
f(\alpha +j)&=(\alpha+j)^p-(\alpha+j)+a\\
&=\alpha^p+j^p-\alpha-j+a\\
&=f(\alpha)=0.
\end{align*}
Here, we used Fermat’s little theorem that $j^a=j$ in $\F_p$.
Thus, $\alpha+j$ is also a root of $f(x)$ for any $j\in \F_p$.

Lemma 2

Lemma 2. The polynomial $f(x)=x^p-x+a$ does not have a root in $\F_p$.

Proof of Lemma 2

If $\alpha$ is a root of $f(x)$ in $\F_p$, then we have
\begin{align*}
0=f(\alpha)=\alpha^p-\alpha+a=a
\end{align*}
since $\alpha^p=\alpha$ in $\F_p$ by Fermat’s little theorem.
However, this contradicts that $a$ is a nonzero element of $\F_p$.

Proof 1 of the irreducibility

Suppose that we have
\[f(x)=g(x)h(x)\] for $g(x), h(x) \in \F_p[x]$.

By Lemma 1, if $\alpha$ is a root of $f(x)$, then $\alpha+j$ is also a root of $f(x)$ for any $j\in \F_p$. Thus, $\alpha + j$ is a root of either $g(x)$ or $h(x)$. From this, we obtain that
\[g(x)=\prod_{j\in I}(x-(\alpha+j)),\] where $I$ is a subset of $\F_p$.

Expanding the product, we see that
\[g(x)=x^n-\sum_{j\in I} (\alpha +j)x^{n-1}+\text{ (lower terms)},\] where $n=|I|$.
Since $g(x) \in \F_p[x]$, the coefficient of $x^{n-1}$ is in $\F_p$. Thus we have
\begin{align*}
\F_p \ni \sum_{j\in I} (\alpha +j)=n\alpha +\sum_{j\in I} j.
\end{align*}

Since $\sum_{j\in I} j\in \F_p$, we deduce that $n \alpha \in \F_p$.
Since by Lemma 2, $\alpha \not \in \F_p$, we must have $n=0$ in $\F_p$.
(Otherwise $n$ is invertible in $\F_p$ and we would get $\alpha \in \F_p$.)
Therefore $n=|I|$ is either $0$ or $p$.
If $n=0$, then $g(x)=1$. If $n=p$, then $h(x)=1$. This implies that $f(x)$ is irreducible over $\F_p$.

Proof 2 of the irreducibility

We give another proof that $f(x)=x^p-x+a$ is irreducible over $\F_p$.

Let $m(x)\in \F_p[x]$ be the minimal polynomial of the root $\alpha$ of $f(x)$.
Then we have $f(x)=m(x)f_1(x)$ for some $f_1(x) \in \F_p[x]$.

If $f_1(x)=1$, then $f(x)=m(x)$ is irreducible as the minimal polynomial is irreducible.
If not, then $f_1(x)$ has some root, and it must be of the form $\alpha+j$ for some $j\in \F_p$ by Lemma 1.
It is straightforward to check that the minimal polynomial of $\alpha+j$ is $m(x-j)$. Thus we can write $f_1(x)=m(x-j)f_2(x)$.

If $f_2(x)=1$, we stop here. If not we iterate the same procedure with $f_2$ as above. Eventually we obtain
\[f(x)=\prod_{j\in I}m(x-j)\] for some subset $I$ of $\F_p$.

Let $n$ be the degree of $m(x)$. Then comparing the degree of both sides, we have
\[p=n|I|.\] Since $p$ is prime, we have either $n=1, |I|=p$, or $n=p$, $|I|=1$.
The former case implies that the minimal polynomial $m(x)$ of $\alpha$ is degree $1$, and hence $\alpha \in \F_p$. However, this cannot happen by Lemma 2.
So we must have $n=p$ and $|I|=1$, which deduce that $f(x)=m(x)$ and $f(x)$ is irreducible over $\F_p$.

Comment.

The polynomial $f(x)=x^p-x+a$ is studied in Artin–Schreier theory.


LoadingAdd to solve later

Sponsored Links

More from my site

  • Degree of an Irreducible Factor of a Composition of PolynomialsDegree of an Irreducible Factor of a Composition of Polynomials Let $f(x)$ be an irreducible polynomial of degree $n$ over a field $F$. Let $g(x)$ be any polynomial in $F[x]$. Show that the degree of each irreducible factor of the composite polynomial $f(g(x))$ is divisible by $n$.   Hint. Use the following fact. Let $h(x)$ is an […]
  • Irreducible Polynomial $x^3+9x+6$ and Inverse Element in Field ExtensionIrreducible Polynomial $x^3+9x+6$ and Inverse Element in Field Extension Prove that the polynomial \[f(x)=x^3+9x+6\] is irreducible over the field of rational numbers $\Q$. Let $\theta$ be a root of $f(x)$. Then find the inverse of $1+\theta$ in the field $\Q(\theta)$.   Proof. Note that $f(x)$ is a monic polynomial and the prime […]
  • $x^3-\sqrt{2}$ is Irreducible Over the Field $\Q(\sqrt{2})$$x^3-\sqrt{2}$ is Irreducible Over the Field $\Q(\sqrt{2})$ Show that the polynomial $x^3-\sqrt{2}$ is irreducible over the field $\Q(\sqrt{2})$.   Hint. Consider the field extensions $\Q(\sqrt{2})$ and $\Q(\sqrt[6]{2})$. Proof. Let $\sqrt[6]{2}$ denote the positive real $6$-th root of of $2$. Then since $x^6-2$ is […]
  • Explicit Field Isomorphism of Finite FieldsExplicit Field Isomorphism of Finite Fields (a) Let $f_1(x)$ and $f_2(x)$ be irreducible polynomials over a finite field $\F_p$, where $p$ is a prime number. Suppose that $f_1(x)$ and $f_2(x)$ have the same degrees. Then show that fields $\F_p[x]/(f_1(x))$ and $\F_p[x]/(f_2(x))$ are isomorphic. (b) Show that the polynomials […]
  • Equation $x_1^2+\cdots +x_k^2=-1$ Doesn’t Have a Solution in Number Field $\Q(\sqrt[3]{2}e^{2\pi i/3})$Equation $x_1^2+\cdots +x_k^2=-1$ Doesn’t Have a Solution in Number Field $\Q(\sqrt[3]{2}e^{2\pi i/3})$ Let $\alpha= \sqrt[3]{2}e^{2\pi i/3}$. Prove that $x_1^2+\cdots +x_k^2=-1$ has no solutions with all $x_i\in \Q(\alpha)$ and $k\geq 1$.   Proof. Note that $\alpha= \sqrt[3]{2}e^{2\pi i/3}$ is a root of the polynomial $x^3-2$. The polynomial $x^3-2$ is […]
  • Prove that any Algebraic Closed Field is InfiniteProve that any Algebraic Closed Field is Infinite Prove that any algebraic closed field is infinite.     Definition. A field $F$ is said to be algebraically closed if each non-constant polynomial in $F[x]$ has a root in $F$. Proof. Let $F$ be a finite field and consider the polynomial \[f(x)=1+\prod_{a\in […]
  • Prove that $\F_3[x]/(x^2+1)$ is a Field and Find the Inverse ElementsProve that $\F_3[x]/(x^2+1)$ is a Field and Find the Inverse Elements Let $\F_3=\Zmod{3}$ be the finite field of order $3$. Consider the ring $\F_3[x]$ of polynomial over $\F_3$ and its ideal $I=(x^2+1)$ generated by $x^2+1\in \F_3[x]$. (a) Prove that the quotient ring $\F_3[x]/(x^2+1)$ is a field. How many elements does the field have? (b) […]
  • Application of Field Extension to Linear CombinationApplication of Field Extension to Linear Combination Consider the cubic polynomial $f(x)=x^3-x+1$ in $\Q[x]$. Let $\alpha$ be any real root of $f(x)$. Then prove that $\sqrt{2}$ can not be written as a linear combination of $1, \alpha, \alpha^2$ with coefficients in $\Q$.   Proof. We first prove that the polynomial […]

You may also like...

2 Responses

  1. Hansi says:

    minor issues:
    In the line with f'(x) you should imo differentiate, as if you were in the Real numbers
    so f'(x)=p*x^(p-^)-1

    In the Proof of Lemma1, second line, there’s a minor error with the sign of the second j, should be -j

Click here to cancel reply.

Please Login to Comment.

This site uses Akismet to reduce spam. Learn how your comment data is processed.

More in Field Theory
Problems and Solutions in Field Theory in Abstract Algebra
Show that Two Fields are Equal: $\Q(\sqrt{2}, \sqrt{3})= \Q(\sqrt{2}+\sqrt{3})$

Show that fields $\Q(\sqrt{2}+\sqrt{3})$ and $\Q(\sqrt{2}, \sqrt{3})$ are equal.  

Close