Skip to content

Commit

Permalink
Review
Browse files Browse the repository at this point in the history
  • Loading branch information
xroblot committed Dec 2, 2024
1 parent 31f190d commit 06b4225
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Analysis/BoxIntegral/UnitPartition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -423,7 +423,7 @@ theorem _root_.tendsto_card_div_pow_atTop_volume (hs₁ : IsBounded s)
· rw [setIntegral_const, smul_eq_mul, mul_one]

private def tendsto_card_div_pow₁ {c : ℝ} (hc : c ≠ 0) :
↑(s ∩ c⁻¹ • L) ≃ ↑(c • s ∩ L) :=
↑(s ∩ c⁻¹ • L) ≃ ↑(c • s ∩ L) :=
Equiv.subtypeEquiv (Equiv.smulRight hc) (fun x ↦ by
simp_rw [Set.mem_inter_iff, Equiv.smulRight_apply, Set.smul_mem_smul_set_iff₀ hc,
← Set.mem_inv_smul_set_iff₀ hc])
Expand Down

0 comments on commit 06b4225

Please sign in to comment.