Skip to content

Commit

Permalink
Replace unnecessary congr with rfl
Browse files Browse the repository at this point in the history
  • Loading branch information
js2357 committed Jul 20, 2024
1 parent 799a4cd commit f365540
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 @@ -854,7 +854,7 @@ private lemma indicator_le : ∀ u ∈ (𝔘₁ k n j).toFinset.filter (x ∈
simp only [𝔘₁, Finset.mem_filter, toFinset_setOf] at hu
apply le_of_le_of_eq hu.1.2.1.1.2
simp only [Finset.coe_filter, mem_toFinset, 𝔐', Finset.card_eq_sum_ones]
refine Finset.sum_congr (by congr) (fun m hm ↦ ?_)
refine Finset.sum_congr rfl (fun m hm ↦ ?_)
simp only [TileLike.le_def, smul_fst, Finset.mem_filter] at hm
simp [hm.2.2.1.1 hx]

Expand Down

0 comments on commit f365540

Please sign in to comment.