Skip to content

Commit

Permalink
Remove unnecessary detail
Browse files Browse the repository at this point in the history
  • Loading branch information
js2357 committed Jul 20, 2024
1 parent 8ccedb0 commit 799a4cd
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Carleson/DiscreteCarleson.lean
Original file line number Diff line number Diff line change
Expand Up @@ -798,7 +798,7 @@ variable (m) (u : 𝔓 X) in
private lemma balls_cover_big_ball : CoveredByBalls (big_ball m u) (defaultA a ^ 9) 0.2 :=
BallsCoverBalls.pow_mul (fun _ ↦ CompatibleFunctions.ballsCoverBalls) (𝒬 m)

private lemma 𝒬_injOn_π”˜m : InjOn (𝒬 (X := X)) (π”˜ k n j x m).toSet :=
private lemma 𝒬_injOn_π”˜m : InjOn 𝒬 (π”˜ k n j x m).toSet :=
fun _ hu _ hu' h ↦ 𝒬_inj h (π“˜_eq_π“˜ hu hu')

private lemma card_π”˜m_le : (π”˜ k n j x m).card ≀ (defaultA a) ^ 9 := by
Expand Down

0 comments on commit 799a4cd

Please sign in to comment.