IMO 2025 Q3 #
Let ℕ+ denote the set of positive integers. A function f : ℕ+ → ℕ+ is said to be bonza if
f a ∣ b ^ a - (f b) ^ (f a) for all positive integers a and b.
Determine the smallest real constant c such that f n ≤ c * n for all bonza functions f and
all positive integers n.
Solution #
We follow solution from https://web.evanchen.cc/exams/IMO-2025-notes.pdf.
We first plug in a = b = n to get the basic constraint ∀ n, f n ∣ n ^ n. Next, one shows that
unless f is the identity, every odd prime must satisfy f p = 1. From here, any odd prime divisor
of f n is ruled out by taking a = n, b = p, so f n is always a power of 2.
Finally, evaluating a = n, b = 3 gives f n ∣ 3 ^ n - 1, and according to the LTE lemma, we have
padicValNat 2 (3 ^ n - 1) = padicValNat 2 n + 2 for Even n. Therefore,
f(n) ≤ 2 ^ (padicValNat 2 n + 2) ≤ 4 * n, so c=4 works.
A matching construction is f n = 1 for Odd n, f 4 = 16, and f n = 2 for other Even n,
which attains the bound, showing the optimal answer is c = 4.