IMO 1998 Q2 #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4. In a competition, there are
a
contestants andb
judges, whereb ≥ 3
is an odd integer. Each judge rates each contestant as either "pass" or "fail". Supposek
is a number such that, for any two judges, their ratings coincide for at mostk
contestants. Prove thatk / a ≥ (b - 1) / (2b)
.
Solution #
The problem asks us to think about triples consisting of a contestant and two judges whose ratings
agree for that contestant. We thus consider the subset A ⊆ C × JJ
of all such incidences of
agreement, where C
and J
are the sets of contestants and judges, and JJ = J × J - {(j, j)}
. We
have natural maps: left : A → C
and right: A → JJ
. We count the elements of A
in two ways: as
the sum of the cardinalities of the fibres of left
and as the sum of the cardinalities of the
fibres of right
. We obtain an upper bound on the cardinality of A
from the count for right
,
and a lower bound from the count for left
. These two bounds combine to the required result.
First consider the map right : A → JJ
. Since the size of any fibre over a point in JJ is bounded
by k
and since |JJ| = b^2 - b
, we obtain the upper bound: |A| ≤ k(b^2-b)
.
Now consider the map left : A → C
. The fibre over a given contestant c ∈ C
is the set of
ordered pairs of (distinct) judges who agree about c
. We seek to bound the cardinality of this
fibre from below. Minimum agreement for a contestant occurs when the judges' ratings are split as
evenly as possible. Since b
is odd, this occurs when they are divided into groups of size
(b-1)/2
and (b+1)/2
. This corresponds to a fibre of cardinality (b-1)^2/2
and so we obtain
the lower bound: a(b-1)^2/2 ≤ |A|
.
Rearranging gives the result.
A triple consisting of contestant together with an ordered pair of judges.
The first judge from an ordered pair of judges.
The second judge from an ordered pair of judges.
The proposition that the judges in an ordered pair are distinct.
The proposition that the judges in an ordered pair agree about a contestant's rating.
The contestant from the triple consisting of a contestant and an ordered pair of judges.
The ordered pair of judges from the triple consisting of a contestant and an ordered pair of judges.
The set of contestants on which two judges agree.
Equations
- imo1998_q2.agreed_contestants r p = finset.filter (λ (c : C), imo1998_q2.judge_pair.agree r p c) finset.univ
All incidences of agreement.
Equations
- imo1998_q2.A r = finset.filter (λ (a : imo1998_q2.agreed_triple C J), imo1998_q2.judge_pair.agree r a.judge_pair a.contestant ∧ a.judge_pair.distinct) finset.univ