Skip to content

Commit

Permalink
chore(Analysis/NormedSpace/PiLp): golf a proof (#11619)
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Mar 24, 2024
1 parent f29c550 commit 971aea7
Showing 1 changed file with 3 additions and 4 deletions.
7 changes: 3 additions & 4 deletions Mathlib/Analysis/NormedSpace/PiLp.lean
Expand Up @@ -395,13 +395,12 @@ attribute [local instance] PiLp.pseudoMetricAux

theorem lipschitzWith_equiv_aux : LipschitzWith 1 (WithLp.equiv p (∀ i, β i)) := by
intro x y
simp_rw [ENNReal.coe_one, one_mul, edist_pi_def, Finset.sup_le_iff, Finset.mem_univ,
forall_true_left, WithLp.equiv_pi_apply]
rcases p.dichotomy with (rfl | h)
· simpa only [ENNReal.coe_one, one_mul, edist_eq_iSup, edist, Finset.sup_le_iff, Finset.mem_univ,
forall_true_left] using le_iSup fun i => edist (x i) (y i)
· simpa only [edist_eq_iSup] using le_iSup fun i => edist (x i) (y i)
· have cancel : p.toReal * (1 / p.toReal) = 1 := mul_div_cancel₀ 1 (zero_lt_one.trans_le h).ne'
rw [edist_eq_sum (zero_lt_one.trans_le h)]
simp only [edist, forall_prop_of_true, one_mul, Finset.mem_univ, Finset.sup_le_iff,
ENNReal.coe_one]
intro i
calc
edist (x i) (y i) = (edist (x i) (y i) ^ p.toReal) ^ (1 / p.toReal) := by
Expand Down

0 comments on commit 971aea7

Please sign in to comment.