Documentation

FormalConjectures.ErdosProblems.«418»

Erdős Problem 418 #

Reference: erdosproblems.com/418

Reviewed by @b-mehta on 2025-05-27

theorem erdos_418 :
{x : | ∃ (n : ), n - n.totient = x}.Infinite True

Are there infinitely many integers not of the form $n - \phi(n)$?

This is true, as shown by Browkin and Schinzel [BrSc95].

[BrSc95] Browkin, J. and Schinzel, A., On integers not of the form {$n-\phi(n)$}. Colloq. Math. (1995), 55-58.

theorem erdos_418.variants.conditional (goldbach : ∀ (n : ), 6 < nEven n∃ (p : ) (q : ), p q Nat.Prime p Nat.Prime q n = p + q) (m : ) (h : Odd m) :
∃ (n : ), m + n.totient = n

It follows from a slight strengthening of the Goldbach conjecture that every odd number can be written as $n - \phi(n)$. In particular, we assume that every even number greater than 6 can be written as the sum of two distinct primes, in contrast to the usual Goldbach conjecture that every even number greater than 2 can be written as the sum of two primes.

theorem erdos_418.variants.sigma :
∃ (S : Set ) (_ : S.HasPosDensity), S {x : | ∃ (n : ), (ArithmeticFunction.sigma 1) n - n = x}

Erdős has shown that a positive density set of integers cannot be written as $\sigma(n) - n$.

[Er73b] Erdős, P., Über die Zahlen der Form $\sigma (n)-n$ und $n-\phi(n)$. Elem. Math. (1973), 83-86.

theorem erdos_418.variants.soln :
{x : | ∃ (k : ), 2 ^ (k + 1) * 509203 = x} {x : | ∃ (n : ), n - n.totient = x}

A solution to erdos_418 was shown by Browkin and Schinzel [BrSc95] by showing that any integer of the form $2^(k + 1)\cdot 509203$ is not of the form $n - \phi(n)$.

[BrSc95] Browkin, J. and Schinzel, A., On integers not of the form {$n-\phi(n)$}. Colloq. Math. (1995), 55-58.

theorem erdos_418.variants.density :
(∃ (S : Set ) (_ : S.HasPosDensity), S {x : | ∃ (n : ), n - n.totient = x}) sorry

It seems to be open whether there is a positive density set of integers not of the form $n - \phi(n)$.