Skip to content

Commit

Permalink
fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn committed Mar 22, 2024
1 parent 57ab23f commit 8204ff6
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
4 changes: 2 additions & 2 deletions Carleson/Carleson.lean
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
import Carleson.Proposition1

open MeasureTheory Measure NNReal Metric Complex Set Function BigOperators Finset
open MeasureTheory Measure NNReal Metric Complex Set Function BigOperators
open scoped ENNReal
noncomputable section
local macro_rules | `($x ^ $y) => `(HPow.hPow $x $y) -- Porting note: See issue lean4#2220
Expand Down Expand Up @@ -90,7 +90,7 @@ lemma sum_Ks {s : Finset ℤ} (hs : nonzeroS D (dist x y) ⊆ s) (hD : 1 < D) (h
norm_cast
suffices : ∑ i in s, ψ (D ^ i * dist x y) = 1
· simp [this]
rw [← sum_subset hs, h3ψ _ h2]
rw [← Finset.sum_subset hs, h3ψ _ h2]
intros
rwa [psi_eq_zero_iff h2ψ h2 hD]

Expand Down
4 changes: 2 additions & 2 deletions README.md
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
# carleson
A (WIP) formalized proof of Carleson's theorem in Lean
# Formalization of a generalized Carleson's theorem
A (WIP) formalized proof of a generalized Carleson's theorem in Lean

## Contribute

Expand Down

0 comments on commit 8204ff6

Please sign in to comment.