Skip to content

Commit

Permalink
fixed notation port to lip section in lp
Browse files Browse the repository at this point in the history
  • Loading branch information
chriscamano committed Jun 16, 2023
1 parent f91fae3 commit 2a52137
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Analysis/NormedSpace/lpSpace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1223,6 +1223,10 @@ end lp

section Lipschitz

local notation "ℓ^∞(" ι ")" => lp (fun i : ι => ℝ) ∞

This comment has been minimized.

Copy link
@tb65536

tb65536 Jun 16, 2023

Collaborator

Does open lp work instead?


open ENNReal

lemma LipschitzWith.uniformly_bounded [PseudoMetricSpace α] (g : α → ι → ℝ) {K : ℝ≥0}
(hg : ∀ i, LipschitzWith K (g · i)) (a₀ : α) (hga₀b : Memℓp (g a₀) ∞) (a : α) :
Memℓp (g a) ∞ := by
Expand Down

0 comments on commit 2a52137

Please sign in to comment.