Skip to content

Commit

Permalink
Lemma 5.1.1 (#78)
Browse files Browse the repository at this point in the history
  • Loading branch information
austinletson authored Jul 15, 2024
1 parent 68d7666 commit 1bc2ab0
Showing 1 changed file with 12 additions and 1 deletion.
13 changes: 12 additions & 1 deletion Carleson/DiscreteCarleson.lean
Original file line number Diff line number Diff line change
Expand Up @@ -476,7 +476,18 @@ lemma third_exception : volume (G₃ (X := X)) ≤ 2 ^ (- 4 : ℤ) * volume G :=

/-- Lemma 5.1.1 -/
lemma exceptional_set : volume (G' : Set X) ≤ 2 ^ (- 2 : ℤ) * volume G :=
sorry
calc volume G'
_ ≤ volume G₁ + volume G₂ + volume G₃ :=
le_add_of_le_add_right (measure_union_le _ G₃) (measure_union_le _ _)
_ ≤ 2 ^ (- 4 : ℤ) * volume G + 2 ^ (- 4 : ℤ) * volume G + 2 ^ (- 4 : ℤ) * volume G :=
add_le_add_three first_exception second_exception third_exception
_ = (3 : ℝ≥0∞) * 2 ^ (-4 : ℤ) * volume G := by ring
_ ≤ 2 ^ (- 2 : ℤ) * volume G :=
have coefficient_inequality : (3 : ℝ≥0∞) * 2 ^ (-4 : ℤ) ≤ (2 : ℝ≥0∞) ^ (-2 : ℤ) := by
change ((3 : ℝ≥0) : ℝ≥0∞) * (2 : ℝ≥0) ^ (-4 : ℤ) ≤ (2 : ℝ≥0) ^ (-2 : ℤ)
repeat rw [← ENNReal.coe_zpow (show (2 : ℝ≥0) ≠ 0 by norm_num)]
rw_mod_cast [← NNReal.coe_le_coe]; norm_num
mul_le_mul_right' coefficient_inequality _

/-! ## Section 5.3 -/

Expand Down

0 comments on commit 1bc2ab0

Please sign in to comment.