Skip to content

Commit 2ba0365

Browse files
Merge branch 'main' into erdos-graffiti-conjecture
2 parents 6cc6655 + 80479cd commit 2ba0365

29 files changed

+916
-36
lines changed
Lines changed: 44 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,44 @@
1+
/-
2+
Copyright 2025 The Formal Conjectures Authors.
3+
4+
Licensed under the Apache License, Version 2.0 (the "License");
5+
you may not use this file except in compliance with the License.
6+
You may obtain a copy of the License at
7+
8+
https://www.apache.org/licenses/LICENSE-2.0
9+
10+
Unless required by applicable law or agreed to in writing, software
11+
distributed under the License is distributed on an "AS IS" BASIS,
12+
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
13+
See the License for the specific language governing permissions and
14+
limitations under the License.
15+
-/
16+
17+
import FormalConjectures.Util.ProblemImports
18+
19+
/-!
20+
# Approximation of Quantum Gates using Lattices
21+
22+
*Reference:* [arxiv/1506.05785](https://arxiv.org/pdf/1506.05785)
23+
_On the Approximation of Quantum Gates using Lattices_
24+
by *Alec Greene and Steven Damelin*
25+
-/
26+
27+
open scoped EuclideanSpace
28+
29+
/-- The integer lattice ℤ⁴ as the ℤ-span of the standard basis in 4-dimensional Euclidean space. -/
30+
scoped[EuclideanSpace] notation "ℤ⁴" => Submodule.span ℤ (Set.range (PiLp.basisFun 2 ℝ (Fin 4)))
31+
32+
instance : IsZLattice ℝ ℤ⁴ := ZSpan.isZLattice _
33+
34+
/--
35+
*Conjecture 3.4*
36+
There exists $0 < \delta < 1$ such that for any $a \in \mathbb{S}^3$,
37+
there exists $b \in \mathbb{Z}^4$ and $k \in \mathbb{Z}$ such that $\|b\| = 5^k$ and
38+
$\langle a, \frac{b}{\|b\|} \rangle \geq 1 - 5^{-\frac{k}{2 - \delta}}.$
39+
-/
40+
@[category research open, AMS 81 11]
41+
theorem conjecture_3_4 : ∃ (δ : ℝ), 0 < δ ∧ δ < 1
42+
∀ (a : EuclideanSpace ℝ (Fin 4)) (ha : ‖a‖ = 1), ∃ (b : ℤ⁴) (k : ℤ), ‖b‖ = 5 ^ k ∧
43+
inner a (‖b‖⁻¹ • b) ≥ 1 - (5 : ℝ) ^ (-k / (2 - δ)) := by
44+
sorry
Lines changed: 38 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,38 @@
1+
/-
2+
Copyright 2025 The Formal Conjectures Authors.
3+
4+
Licensed under the Apache License, Version 2.0 (the "License");
5+
you may not use this file except in compliance with the License.
6+
You may obtain a copy of the License at
7+
8+
https://www.apache.org/licenses/LICENSE-2.0
9+
10+
Unless required by applicable law or agreed to in writing, software
11+
distributed under the License is distributed on an "AS IS" BASIS,
12+
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
13+
See the License for the specific language governing permissions and
14+
limitations under the License.
15+
-/
16+
17+
import FormalConjectures.Util.ProblemImports
18+
19+
/-!
20+
# Erdős Problem 128
21+
22+
*Reference:* [erdosproblems.com/128](https://www.erdosproblems.com/128)
23+
-/
24+
25+
variable {V : Type*} {G : SimpleGraph V} [Fintype V]
26+
27+
/--
28+
Let G be a graph with n vertices such that every subgraph on ≥ $n/2$
29+
vertices has more than $n^2/50$ edges. Must G contain a triangle?
30+
-/
31+
@[category research open, AMS 5]
32+
theorem erdos_128 :
33+
((∀ (G' : G.Subgraph) [Fintype G'.verts] [Fintype G'.edgeSet],
34+
letI n := Fintype.card V;
35+
2 * G'.verts.toFinset.card ≥ n →
36+
50 * G'.edgeSet.toFinset.card > n^2) → ¬ (G.CliqueFree 3))
37+
↔ answer(sorry) := by
38+
sorry
Lines changed: 114 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,114 @@
1+
/-
2+
Copyright 2025 The Formal Conjectures Authors.
3+
4+
Licensed under the Apache License, Version 2.0 (the "License");
5+
you may not use this file except in compliance with the License.
6+
You may obtain a copy of the License at
7+
8+
https://www.apache.org/licenses/LICENSE-2.0
9+
10+
Unless required by applicable law or agreed to in writing, software
11+
distributed under the License is distributed on an "AS IS" BASIS,
12+
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
13+
See the License for the specific language governing permissions and
14+
limitations under the License.
15+
-/
16+
17+
import FormalConjectures.Util.ProblemImports
18+
19+
/-!
20+
# Erdős Problem 141
21+
22+
*References:*
23+
- [erdosproblems.com/141](https://www.erdosproblems.com/141)
24+
- [Wikipedia](https://en.wikipedia.org/wiki/Primes_in_arithmetic_progression#Consecutive_primes_in_arithmetic_progression)
25+
-/
26+
27+
/--
28+
The predicate that a set `s` consists of `l` consecutive primes (possibly infinite).
29+
This predicate does not assert a specific value for the first term.
30+
-/
31+
def Set.IsPrimeProgressionOfLength (s : Set ℕ) (l : ℕ∞) : Prop :=
32+
∃ a, ENat.card s = l ∧ s = {(a + n).nth Nat.Prime | (n : ℕ) (_ : n < l)}
33+
34+
open Nat
35+
36+
/--
37+
The first three odd primes are an example of three consecutive primes.
38+
-/
39+
@[category test, AMS 5 11]
40+
theorem first_three_odd_primes : ({3, 5, 7} : Set ℕ).IsPrimeProgressionOfLength 3 := by
41+
use 1
42+
constructor
43+
· aesop
44+
· norm_num [exists_lt_succ, or_assoc, eq_comm, Set.insert_def,
45+
show (2).nth Nat.Prime = 5 from nth_count prime_five,
46+
show (3).nth Nat.Prime = 7 from Nat.nth_count (by decide : (7).Prime)]
47+
48+
/--
49+
The predicate that a set `s` is both an arithmetic progression of length `l` and a progression
50+
of `l` consecutive primes.
51+
-/
52+
def Set.IsAPAndPrimeProgressionOfLength (s : Set ℕ) (l : ℕ) :=
53+
s.IsAPOfLength l ∧ s.IsPrimeProgressionOfLength l
54+
55+
/--
56+
There are 3 consecutive primes in arithmetic progression.
57+
-/
58+
@[category test, AMS 5 11]
59+
example : ∃ (s : Set ℕ), s.IsAPAndPrimeProgressionOfLength 3 := by
60+
use {3, 5, 7}
61+
constructor
62+
· use 3, 2
63+
unfold Set.IsAPOfLengthWith
64+
constructor
65+
· aesop
66+
· norm_num [exists_lt_succ, or_assoc, eq_comm, Set.insert_def]
67+
· exact first_three_odd_primes
68+
69+
/--
70+
Let $k≥3$. Are there $k$ consecutive primes in arithmetic progression?
71+
-/
72+
@[category research open, AMS 5 11]
73+
theorem erdos_141 : (∀ k ≥ 3, ∃ (s : Set ℕ), s.IsAPAndPrimeProgressionOfLength k)
74+
↔ answer(sorry) := by
75+
sorry
76+
77+
/--
78+
The existence of such progressions has been verified for $k≤10$.
79+
-/
80+
@[category research solved, AMS 5 11]
81+
theorem erdos_141.variant.first_cases :
82+
(∀ k ≥ 3, k ≤ 10 → ∃ (s : Set ℕ), s.IsAPAndPrimeProgressionOfLength k) := by
83+
sorry
84+
85+
/--
86+
Are there $11$ consecutive primes in arithmetic progression?
87+
-/
88+
@[category research open, AMS 5 11]
89+
theorem erdos_141.variant.eleven : (∃ (s : Set ℕ), s.IsAPAndPrimeProgressionOfLength 11)
90+
↔ answer(sorry) := by
91+
sorry
92+
93+
/--
94+
The set of arithmetic progressions of consecutive primes of length $k$.
95+
-/
96+
def consecutivePrimeArithmeticProgressions (k : ℕ) : Set (Set ℕ) :=
97+
{s | s.IsAPAndPrimeProgressionOfLength k}
98+
99+
/--
100+
It is open, even for $k=3$, whether there are infinitely many such progressions.
101+
-/
102+
@[category research open, AMS 5 11]
103+
theorem erdos_141.variant.infinite_three :
104+
(consecutivePrimeArithmeticProgressions 3).Infinite ↔ answer(sorry) :=
105+
sorry
106+
107+
/--
108+
Fix a $k \geq 3$. Is it true that there are infinitely many arithmetic prime progressions of length $k$?
109+
-/
110+
@[category research open, AMS 5 11]
111+
theorem erdos_141.variant.infinite_general_case (k : ℕ) (hk : k ≥ 3) :
112+
(consecutivePrimeArithmeticProgressions k).Infinite ↔ answer(sorry) :=
113+
sorry
114+

FormalConjectures/ErdosProblems/168.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -66,8 +66,8 @@ Sanity check: if `S` is a maximal non ternary subset of `{1,..., N}` then `F N`
6666
cardinality of `S`
6767
-/
6868
@[category API, AMS 5 11]
69-
lemma F_eq_card (N : ℕ) (S : Finset ℕ) (hS : S ⊆ Finset.Icc 1 N)
70-
(hS' : NonTernary S) (hS'' : ∀ T, T ⊆ Finset.Icc 1 N → NonTernary T → S ⊆ T → T = S) :
69+
lemma F_eq_card (N : ℕ) (S : Finset ℕ) (hS : S ⊆ Finset.Icc 1 N) (hS' : NonTernary S)
70+
(hS'' : ∀ T, T ⊆ Finset.Icc 1 N → NonTernary T → S.card ≤ T.card → T.card = S.card) :
7171
F N = S.card := by
7272
sorry
7373

Lines changed: 47 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,47 @@
1+
/-
2+
Copyright 2025 The Formal Conjectures Authors.
3+
4+
Licensed under the Apache License, Version 2.0 (the "License");
5+
you may not use this file except in compliance with the License.
6+
You may obtain a copy of the License at
7+
8+
https://www.apache.org/licenses/LICENSE-2.0
9+
10+
Unless required by applicable law or agreed to in writing, software
11+
distributed under the License is distributed on an "AS IS" BASIS,
12+
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
13+
See the License for the specific language governing permissions and
14+
limitations under the License.
15+
-/
16+
17+
import FormalConjectures.Util.ProblemImports
18+
19+
/-!
20+
# Erdős Problem 200
21+
22+
*Reference:* [erdosproblems.com/200](https://www.erdosproblems.com/200)
23+
-/
24+
25+
open Filter Real
26+
27+
/--
28+
The length of the longest arithmetic progression of primes in $\{1,\ldots,n\}$.
29+
-/
30+
noncomputable def longestPrimeArithmeticProgressions (n : ℕ) : ℕ :=
31+
sSup {(k : ℕ) | ∃ s ⊆ Set.Icc 1 n, s.IsAPOfLength k ∧ ∀ m ∈ s, m.Prime}
32+
33+
/--
34+
Does the longest arithmetic progression of primes in $\{1,\ldots,N\}$ have length $o(\log N)$?
35+
-/
36+
@[category research open, AMS 5 11]
37+
theorem erdos_200 : (fun n => (longestPrimeArithmeticProgressions n : ℝ))
38+
=o[atTop] (fun n => log n) ↔ answer(sorry) := by
39+
sorry
40+
41+
/--
42+
It follows from the prime number theorem that such a progression has length $\leq(1+o(1))\log N$.
43+
-/
44+
@[category research solved, AMS 5 11]
45+
theorem erdos_200.variants.upper : ∃ (o : ℕ → ℝ) (_ : o =o[atTop] (1 : ℕ → ℝ)),
46+
∀ n, longestPrimeArithmeticProgressions n ≤ (1 + o n) * log n := by
47+
sorry
Lines changed: 57 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,57 @@
1+
/-
2+
Copyright 2025 The Formal Conjectures Authors.
3+
4+
Licensed under the Apache License, Version 2.0 (the "License");
5+
you may not use this file except in compliance with the License.
6+
You may obtain a copy of the License at
7+
8+
https://www.apache.org/licenses/LICENSE-2.0
9+
10+
Unless required by applicable law or agreed to in writing, software
11+
distributed under the License is distributed on an "AS IS" BASIS,
12+
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
13+
See the License for the specific language governing permissions and
14+
limitations under the License.
15+
-/
16+
17+
import FormalConjectures.Util.ProblemImports
18+
19+
/-!
20+
# Erdős Problem 208
21+
*Reference:* [erdosproblems.com/208](https://www.erdosproblems.com/208)
22+
-/
23+
24+
open Filter Real
25+
26+
/-- The sequence of squarefree numbers, denoted by `s` as in Erdős problem 208. -/
27+
noncomputable def erdos208.s : ℕ → ℕ := Nat.nth Squarefree
28+
29+
open erdos208
30+
31+
/--
32+
Let $s_1 < s_2 < ⋯$ be the sequence of squarefree numbers. Is it true that
33+
for any $ϵ > 0$ and large $n$, $s_{n+1} − s_n ≪_ϵ s_n^ε$?
34+
-/
35+
@[category research open, AMS 11]
36+
theorem erdos_208.i :
37+
(∀ ε > (0 : ℝ), (fun n => (s (n + 1) - s n : ℝ)) =O[atTop] (fun n => (s n : ℝ)^ε)) ↔
38+
answer(sorry) := by sorry
39+
40+
/--
41+
Let $s_1 < s_2 < ⋯$ be the sequence of squarefree numbers. Is it true that
42+
$s_{n + 1} - s_n ≤ (1 + o(1)) * (\pi^2 / 6) * log (s_n) / log (log (s_n))$?
43+
-/
44+
@[category research open, AMS 11]
45+
theorem erdos_208.ii :
46+
(∃ (c : ℕ → ℝ), (c =o[atTop] (1 : ℕ → ℝ)) ∧ ∀ᶠ n in atTop,
47+
s (n + 1) - s n ≤ (1 + (c n)) * (π^2 / 6) * log (s n) / log (log (s n))) ↔ answer(sorry) := by
48+
sorry
49+
50+
/--
51+
In [Er79] Erdős says perhaps $s_{n+1} − s_n ≪ log s_n$, but he is 'very doubtful'.
52+
53+
[Er79] Erdős, Paul, __Some unconventional problems in number theory__. Math. Mag. (1979), 67-70.
54+
-/
55+
@[category research open, AMS 11]
56+
theorem erdos_208.variants.log_bound :
57+
(fun n ↦ (s (n + 1) - s n : ℝ)) =O[atTop] fun n ↦ log (s n) := by sorry

FormalConjectures/ErdosProblems/245.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -44,7 +44,7 @@ The answer is yes, proved by Freiman [Fr73].
4444
@[category research solved, AMS 5 11]
4545
theorem erdos_245 :
4646
(∀ (A : Set ℕ), A.Infinite → Tendsto (fun N => (A.bdd N |>.ncard : ℝ) / N) atTop (𝓝 0) →
47-
3 ≤ limsup (fun N => ((A + A).bdd N |>.ncard : ) / (A.bdd N).ncard) atTop) ↔ answer(True) := by
47+
3 ≤ limsup (fun N => ((A + A).bdd N |>.ncard : EReal) / (A.bdd N).ncard) atTop) ↔ answer(True) := by
4848
sorry
4949

5050
/--
@@ -73,5 +73,5 @@ $$
7373
@[category research solved, AMS 5 11]
7474
theorem erdos_245.variants.two (A : Set ℕ) (h_inf : A.Infinite)
7575
(hf : Tendsto (fun N => (A.bdd N |>.ncard : ℝ) / N) atTop (𝓝 0)) :
76-
2 ≤ limsup (fun N => ((A + A).bdd N |>.ncard : ) / (A.bdd N).ncard) atTop := by
76+
2 ≤ limsup (fun N => ((A + A).bdd N |>.ncard : EReal) / (A.bdd N).ncard) atTop := by
7777
sorry
Lines changed: 34 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,34 @@
1+
/-
2+
Copyright 2025 The Formal Conjectures Authors.
3+
4+
Licensed under the Apache License, Version 2.0 (the "License");
5+
you may not use this file except in compliance with the License.
6+
You may obtain a copy of the License at
7+
8+
https://www.apache.org/licenses/LICENSE-2.0
9+
10+
Unless required by applicable law or agreed to in writing, software
11+
distributed under the License is distributed on an "AS IS" BASIS,
12+
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
13+
See the License for the specific language governing permissions and
14+
limitations under the License.
15+
-/
16+
17+
import FormalConjectures.Util.ProblemImports
18+
19+
/-!
20+
# Erdős Problem 249
21+
22+
*Reference:* [erdosproblems.com/249](https://www.erdosproblems.com/249)
23+
-/
24+
25+
open scoped Nat
26+
27+
/--
28+
Is
29+
$$\sum_{n} \frac{φ(n)}{2^n}$$
30+
irrational? Here $\phi$ is the Euler totient function.
31+
-/
32+
@[category research open, AMS 11]
33+
theorem erdos_249 : Irrational (∑' n : ℕ, (φ n) / (2 ^ n)) ↔ answer(sorry) := by
34+
sorry

0 commit comments

Comments
 (0)