Skip to content

Commit

Permalink
WIP
Browse files Browse the repository at this point in the history
  • Loading branch information
gdahia committed Sep 26, 2024
1 parent 0f1c1fd commit 262fd17
Showing 1 changed file with 16 additions and 2 deletions.
18 changes: 16 additions & 2 deletions FurstenbergSarkozy/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,21 @@ lemma square_difference_free_set_has_zero_countOfSquares (n : ℕ) (S : Finset
right
exact if_neg (squareDifferenceFree (r + h) x xInS)

lemma uniform_δ_indicator_has_sqr_δ_density_of_countOfSquares
(n : ℕ) (δ : unitInterval) : countOfSquares n (δ • (range n).indicator) = δ ^ 2 * n ^ 2 := by
dsimp [countOfSquares, generalizedCountOfSquares, indicator, piecewise, id']
norm_cast
simp
have : (range (n - ⌈ ((n : ℝ) ^ (1/3 : ℝ)) ⌉₊)) ⊆ (range n) := range_subset.mpr (by omega)
-- apply sum_subset this ?h
sorry

-- approach should be the following: do cases. if we have a single square difference in S, then we are done.
-- otherwise, we can go to a denser subset by the density increment argument
-- and we show that recursively calling furstenberg_sarkozy terminates because δ increases
-- and is at most one

theorem furstenberg_sarkozy :
α : ℝ, ∃ n₀ : ℕ, ∀ n : ℕ, ∀ S ⊆ (range n),
n ≥ n₀ ∧ S.card ≥ α * n → ∃ d : ℕ, ∃ a ∈ S, a + d ^ 2 ∈ S :=
δ : ℝ, ∃ n₀ : ℕ, ∀ n : ℕ, ∀ S ⊆ (range n),
n ≥ n₀ ∧ S.card ≥ δ * n → ∃ d : ℕ, ∃ a ∈ S, a + d ^ 2 ∈ S :=
sorry

0 comments on commit 262fd17

Please sign in to comment.