Difference between revisions of "1974 IMO Problems/Problem 6"
Durianaops (talk | contribs) (Created page with "==Problem== Let <math>P</math> be a non-constant polynomial with integer coefficients. If <math>n(P)</math> is the number of distinct integers <math>k</math> such that <math>(...") |
|||
| (9 intermediate revisions by 2 users not shown) | |||
| Line 1: | Line 1: | ||
==Problem== | ==Problem== | ||
| + | |||
Let <math>P</math> be a non-constant polynomial with integer coefficients. If <math>n(P)</math> is the number of distinct integers <math>k</math> such that <math>(P(k))^2=1,</math> prove that <math>n(P)-\deg(P)\le2,</math> where <math>\deg(P)</math> denotes the degree of the polynomial <math>P.</math> | Let <math>P</math> be a non-constant polynomial with integer coefficients. If <math>n(P)</math> is the number of distinct integers <math>k</math> such that <math>(P(k))^2=1,</math> prove that <math>n(P)-\deg(P)\le2,</math> where <math>\deg(P)</math> denotes the degree of the polynomial <math>P.</math> | ||
| + | |||
==Solution== | ==Solution== | ||
| − | {{solution}} | + | |
| + | Lemma: Let <math>P(x)</math> be a polynomial with integer coefficients which is not constant. Then if <math>P(x)</math> obtains <math>1</math> (or <math>-1</math>) as its values for at least four times then <math>P(x)\neq -1</math> ( or <math>P(x)\neq 1</math>) for all <math>x</math>. | ||
| + | Proof. Assume that <math>P(a)=P(b)=P(c)=P(d)=1</math> for <math>a,b,c,d</math> distince. Then if there's <math>u</math> which <math>P(u)=-1</math> then <math>2=P(a)-P(u)=...</math> so <math>P(x)-P(u)-2=(x-a)(x-b)(x-c)(x-d)Q(x)</math> where <math>Q(x)</math> is a polynomial with the integer coefficients! So | ||
| + | <math>-2=(u-a)(u-b)(u-c)(u-d)Q(u)</math> which is impossible cause <math>-2</math> can not presents as product of more than three distince numbers! This proved the lemma! | ||
| + | |||
| + | Back to our problem: For convinet put <math>m=n(P)</math> and <math>n=\deg P</math>. Firstly if <math>n\leq 2</math> then <math>m-n\leq2</math>. Assume <math>n\geq3</math>. If equation <math>P(x)=1</math> with more than three integer points (ie.. at least <math>4</math>) then equation <math>(P(x))^2=1</math> implies <math>P(x)=1</math> so <math>m\leq n</math>, ie... <math>m-n\leq 0\leq2</math>. The same case for equation <math>P(x)=-1</math>. So <math>m\leq 6</math>. If <math>n\geq4</math> then <math>m-n\leq 6-n\leq 2</math>. Now assume that <math>n=3</math>. In this case if <math>m\leq 5</math> then <math>m-n\leq 2</math>. | ||
| + | |||
| + | So let us show that <math>m<6</math>. In fact if <math>m=6</math> then <math>P(x)-1=0</math> has three integers distince roots, and the same for <math>P(x)+1=0</math>. So | ||
| + | <math>P(x)-1=k_1(x-a_1)(x-a_2)(x-a_3)</math> and <math>P(x)+1=k_2(x-b_1)(x-b_2)(x-b_3)</math> where <math>a_i</math> distince and <math>b_j</math> distince and all with <math>k_1,k_2</math> are integers! Then | ||
| + | <math>k_2(x-b_1)(x-b_2)(x-b_3)-k_1(x-a_1)(x-a_2)(x-a_3)=2</math> for all <math>x</math>. So <math>k_1=k_2=k</math>. | ||
| + | Finally, we have | ||
| + | <math>2=k(a_i-b_1)(a_i-b_2)(a_i-b_3)</math> for <math>i=1,2,3</math> and because that <math>\pm1</math> can not presents as products of three distince numbers so <math>k=\pm1</math>, we may assume <math>k=1</math>. Because <math>2=(-2)\cdot 1\cdot -1</math> so | ||
| + | <math>\{-2,1,-1\}=\{a_i-b_1,a_i-b_2,a_i-b_3\}</math> | ||
| + | This means <math>3a_i-(b_1+b_2+b_3)=-2+1-1=-2</math>. So we must have <math>3a_1=3a_2=3a_3</math> which follows <math>a_1=a_2=a_3</math>, which contracts!. So <math>m\leq 5</math> and we're done. | ||
| + | |||
| + | The above solution was posted and copyrighted by pluricomplex. | ||
| + | |||
| + | |||
| + | ==Remarks (added by pf02, October 2025)== | ||
| + | |||
| + | <math>\mathbf{1.}</math> The solution above is written very sloppily and | ||
| + | badly, it could use substantial editing. However, the proof is | ||
| + | understandable and correct, and I will refrain from rewriting it. | ||
| + | |||
| + | It is interesting to note that it actually proves substantially | ||
| + | more than the problem asked. It proves the following two | ||
| + | statements: | ||
| + | |||
| + | <math>\mathbf{a.}</math> If one of the equations <math>P(x) - 1 = 0</math> and | ||
| + | <math>P(x) + 1 = 0</math> has <math>\ge 4</math> integer, distinct solutions, then | ||
| + | the other has no integer solutions. | ||
| + | |||
| + | <math>\mathbf{b.}</math> If both equations <math>P(x) - 1 = 0</math> and | ||
| + | <math>P(x) + 1 = 0</math> have integer solutions then <math>n(P) \le 5</math>. | ||
| + | |||
| + | The statement of the original problem is a trivial consequence | ||
| + | of these statements (as I will show later). | ||
| + | |||
| + | <math>\mathbf{2.}</math> This problem is in fact very easy. It is made | ||
| + | difficult artificially, by hiding the essence of the description | ||
| + | of the distinct, integer solutions of <math>P(x) - 1 = 0</math> and | ||
| + | <math>P(x) + 1 = 0</math>. The essence is hidden behind a more general | ||
| + | sounding (and in some sense artificial) statement. Had it been | ||
| + | formulated to express the essence of the description of the | ||
| + | distinct, integer roots of <math>P(x) - 1 = 0</math> and <math>P(x) + 1 = 0</math>, | ||
| + | the problem would have been much less intimidating, and much | ||
| + | easier, because the facts would have pointed towards a solution. | ||
| + | |||
| + | Here is a reformulation the problem: | ||
| + | |||
| + | <math>\mathbf{Problem\ 2\ (a\ better\ version\ of\ the\ problem)}</math> | ||
| + | Let <math>P(x)</math> be a polynomial with integer coefficients. Let | ||
| + | <math>m_1 =</math> the number of distinct integer roots of <math>P(x) - 1 = 0</math>, | ||
| + | and <math>m_2 =</math> the number of distinct integer roots of <math>P(x) + 1 = 0</math>. | ||
| + | If both <math>m_1 \ge 1, m_2 \ge 1</math> then <math>n(P) = m = m_1 + m_2 \le 4</math>. | ||
| + | |||
| + | |||
| + | ==Solution 2 (solution of the better problem)== | ||
| + | |||
| + | If <math>\deg(P) = 1</math> or <math>\deg(P) = 2</math> the statement is obviously true. | ||
| + | So, assume <math>\deg(P) \ge 3</math>. | ||
| + | |||
| + | Let <math>M_1 = \{a_1 < \dots < a_{m_1}\}</math> be the integer, distinct solutions | ||
| + | of <math>P(x) - 1 = 0</math>, and let <math>M_2 = \{b_1 < \dots < b_{m_2}\}</math> be the | ||
| + | integer, distinct solutions of <math>P(x) + 1 = 0</math>. Denote | ||
| + | <math>M = \{s_1 < \dots < s_m\}</math> the union <math>M_1 \cup M_2</math> arranged in | ||
| + | increasing order. Thus each <math>s_i</math> could be an element <math>a_j \in M_1</math> | ||
| + | or an element <math>b_k \in M_2</math>. We will think of the sequence <math>M</math> as a | ||
| + | sequence of <math>a</math>'s and <math>b</math>'s. | ||
| + | |||
| + | Let <math>a</math> satisfy <math>P(a) - 1 = 0</math> and <math>b</math> satisfy <math>P(b) + 1 = 0</math>. Then | ||
| + | <math>a - b \in \{-2, -1, 1, 2\}</math>, in other words <math>|a - b| = 1</math> or <math>|a - b| = 2</math>. | ||
| + | Indeed, <math>P(a) - P(b) = (a - b) Q</math> for some integer <math>Q</math>. From | ||
| + | <math>P(a) - P(b) = 2</math> it follows <math>(a - b) Q = 2</math>, so <math>(a - b)</math> must be a divisor | ||
| + | of <math>2</math>. We paraphrase this by saying that any solution of <math>P(x) - 1 = 0</math> | ||
| + | and any solution of <math>P(x) + 1 = 0</math> are at distance at most <math>2</math>. | ||
| + | |||
| + | In terms of looking at <math>M</math> as a sequence of <math>a</math>'s and <math>b</math>'s, given that | ||
| + | all the <math>s_i</math>'s are distinct, this tells us that in terms of the distance | ||
| + | in the counting (or indexing) in the sequence, any <math>b</math> is at most two away | ||
| + | from any <math>a</math>, and any <math>a</math> is at most <math>2</math> away from any <math>b</math>. In other words, | ||
| + | if we have an <math>a</math>, then at most two entries to the right and two entries to | ||
| + | the left are <math>b</math>'s, and, if we have a <math>b</math>, then at most two entries to the | ||
| + | right and two entries to the left are <math>a</math>'s. | ||
| + | |||
| + | It follows that <math>M</math> can not have <math>6</math> (or more) elements. | ||
| + | |||
| + | Indeed, assume that <math>M</math> has <math>6</math> elements | ||
| + | <math>M = \{s_1 < s_2 < s_3 < s_4 < s_5 < s_6\}</math> and assume <math>s_1</math> is an <math>a</math>. | ||
| + | Then <math>s_4, s_5, s_6</math> must be <math>a</math>'s. Since <math>s_6</math> is an <math>a</math>, <math>s_2, s_3</math> | ||
| + | must be <math>a</math>'s. It follows that all <math>s_i</math>'s are <math>a</math>'s, which is a | ||
| + | contradiction since we assumed we have at least one <math>b</math>. | ||
| + | |||
| + | <math>\mathbf{Note}</math> The statement of the original problem follows trivially | ||
| + | from what we proved so far. Indeed, if only one of <math>P(x) - 1 = 0</math> and | ||
| + | <math>P(x) + 1 = 0</math> has integer roots, then <math>n(P) \le d < d + 2</math>. If <math>\deg(P)</math> | ||
| + | is <math>1</math> or <math>2</math>, then <math>n(P) \le 2, 4</math> respectively, which is less than <math>d + 2</math>. | ||
| + | If the degree <math>d = \deg(P) \ge 3</math> then <math>n(P) = m \le 5 \le d + 2</math>. | ||
| + | |||
| + | Let us prove the stronger bound <math>m = m_1 + m_2 \le 4</math>. | ||
| + | |||
| + | Assume that <math>m = m_1 + m_2 = 5</math>. Then we have that <math>m_1, m_2</math> are <math>4</math> | ||
| + | and <math>1</math> (in some order), or <math>m_1, m_2</math> are <math>3</math> and <math>2</math> (in some order). | ||
| + | |||
| + | Assume <math>m_1 = 4, m_2 = 1</math>. This is impossible because of the argument | ||
| + | from the first solution. (Repeat the argument | ||
| + | for the sake of completeness: Assume | ||
| + | <math>P(a_1) = P(a_2) = P(a_3) = P(a_4) = 1</math> and <math>P(b_1) = -1</math>. | ||
| + | Then <math>P(x) = (x - a_1)(x - a_2)(x - a_3)(x - a_4) Q(x) + 1</math> | ||
| + | with <math>Q(x)</math> having integer coefficients. Substituting <math>x = b_1</math> | ||
| + | we have <math>(b_1 - a_1)(b_1 - a_2)(b_1 - a_3)(b_1 - a_4) Q(b_1) = -2</math>. | ||
| + | It follows that the values of the four factors <math>(b_1 - a_i)</math> must | ||
| + | be in <math>\{-2, -1, 1, 2\}</math>. Since they are distinct, they must be | ||
| + | exactly these four values. Then | ||
| + | <math>(b_1 - a_1)(b_1 - a_2)(b_1 - a_3)(b_1 - a_4) Q(b_1)</math> will be | ||
| + | a multiple of 4, and it can not equal <math>-2</math>.) | ||
| + | |||
| + | Now assume <math>m_1 = 3, m_2 = 2</math>. Looking again at | ||
| + | <math>M = \{s_1 < s_2 < s_3 < s_4 < s_5\}</math> as a sequence of <math>a</math>'s and <math>b</math>'s, | ||
| + | assume that <math>s_1</math> is an <math>a</math>. Then <math>s_4, s_5</math> must be <math>a</math>'s. If <math>s_5</math> | ||
| + | is an <math>a</math>, then <math>s_2</math> must be an <math>a</math>. Depending on <math>s_3</math>, either | ||
| + | <math>M</math> has only <math>a</math>'s, which is impossible, or <math>M = \{a, a, b, a, a\}</math>. | ||
| + | This would put us in the case <math>m_1 = 4, m_2 = 1</math>, which is a | ||
| + | contradiction. | ||
| + | |||
| + | The assumption <math>m = m_1 + m_2 = 5</math> led to a contradiction, so <math>m \le 4</math>. | ||
| + | |||
| + | [Solution by pf02, October 2025] | ||
| + | |||
| + | |||
| + | The original thread for this problem can be found here: [https://aops.com/community/p364890] | ||
==See Also== | ==See Also== | ||
{{IMO box|year=1974|num-b=5|after=Last Question}} | {{IMO box|year=1974|num-b=5|after=Last Question}} | ||
| − | [[Category:Olympiad | + | [[Category:Olympiad Algebra Problems]] |
Latest revision as of 00:12, 29 October 2025
Contents
Problem
Let
be a non-constant polynomial with integer coefficients. If
is the number of distinct integers
such that
prove that
where
denotes the degree of the polynomial
Solution
Lemma: Let
be a polynomial with integer coefficients which is not constant. Then if
obtains
(or
) as its values for at least four times then
( or
) for all
.
Proof. Assume that
for
distince. Then if there's
which
then
so
where
is a polynomial with the integer coefficients! So
which is impossible cause
can not presents as product of more than three distince numbers! This proved the lemma!
Back to our problem: For convinet put
and
. Firstly if
then
. Assume
. If equation
with more than three integer points (ie.. at least
) then equation
implies
so
, ie...
. The same case for equation
. So
. If
then
. Now assume that
. In this case if
then
.
So let us show that
. In fact if
then
has three integers distince roots, and the same for
. So
and
where
distince and
distince and all with
are integers! Then
for all
. So
.
Finally, we have
for
and because that
can not presents as products of three distince numbers so
, we may assume
. Because
so
This means
. So we must have
which follows
, which contracts!. So
and we're done.
The above solution was posted and copyrighted by pluricomplex.
Remarks (added by pf02, October 2025)
The solution above is written very sloppily and
badly, it could use substantial editing. However, the proof is
understandable and correct, and I will refrain from rewriting it.
It is interesting to note that it actually proves substantially more than the problem asked. It proves the following two statements:
If one of the equations
and
has
integer, distinct solutions, then
the other has no integer solutions.
If both equations
and
have integer solutions then
.
The statement of the original problem is a trivial consequence of these statements (as I will show later).
This problem is in fact very easy. It is made
difficult artificially, by hiding the essence of the description
of the distinct, integer solutions of
and
. The essence is hidden behind a more general
sounding (and in some sense artificial) statement. Had it been
formulated to express the essence of the description of the
distinct, integer roots of
and
,
the problem would have been much less intimidating, and much
easier, because the facts would have pointed towards a solution.
Here is a reformulation the problem:
Let
be a polynomial with integer coefficients. Let
the number of distinct integer roots of
,
and
the number of distinct integer roots of
.
If both
then
.
Solution 2 (solution of the better problem)
If
or
the statement is obviously true.
So, assume
.
Let
be the integer, distinct solutions
of
, and let
be the
integer, distinct solutions of
. Denote
the union
arranged in
increasing order. Thus each
could be an element
or an element
. We will think of the sequence
as a
sequence of
's and
's.
Let
satisfy
and
satisfy
. Then
, in other words
or
.
Indeed,
for some integer
. From
it follows
, so
must be a divisor
of
. We paraphrase this by saying that any solution of
and any solution of
are at distance at most
.
In terms of looking at
as a sequence of
's and
's, given that
all the
's are distinct, this tells us that in terms of the distance
in the counting (or indexing) in the sequence, any
is at most two away
from any
, and any
is at most
away from any
. In other words,
if we have an
, then at most two entries to the right and two entries to
the left are
's, and, if we have a
, then at most two entries to the
right and two entries to the left are
's.
It follows that
can not have
(or more) elements.
Indeed, assume that
has
elements
and assume
is an
.
Then
must be
's. Since
is an
,
must be
's. It follows that all
's are
's, which is a
contradiction since we assumed we have at least one
.
The statement of the original problem follows trivially
from what we proved so far. Indeed, if only one of
and
has integer roots, then
. If
is
or
, then
respectively, which is less than
.
If the degree
then
.
Let us prove the stronger bound
.
Assume that
. Then we have that
are
and
(in some order), or
are
and
(in some order).
Assume
. This is impossible because of the argument
from the first solution. (Repeat the argument
for the sake of completeness: Assume
and
.
Then
with
having integer coefficients. Substituting
we have
.
It follows that the values of the four factors
must
be in
. Since they are distinct, they must be
exactly these four values. Then
will be
a multiple of 4, and it can not equal
.)
Now assume
. Looking again at
as a sequence of
's and
's,
assume that
is an
. Then
must be
's. If
is an
, then
must be an
. Depending on
, either
has only
's, which is impossible, or
.
This would put us in the case
, which is a
contradiction.
The assumption
led to a contradiction, so
.
[Solution by pf02, October 2025]
The original thread for this problem can be found here: [1]
See Also
| 1974 IMO (Problems) • Resources | ||
| Preceded by Problem 5 |
1 • 2 • 3 • 4 • 5 • 6 | Followed by Last Question |
| All IMO Problems and Solutions | ||