Skip to content

Commit

Permalink
feat: port Analysis.NormedSpace.LpSpace (#4465)
Browse files Browse the repository at this point in the history
Notes [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/!4.234465.20.60lp.60) :
1. There are both `CoeOut` and `CoeFun` instances for `lp E p`. This is consistent with mathlib3, but it seems strange and I would expect it to cause problems.
2. It seems there is some defeq abuse (identifiying `PreLp E` with `∀ i, E i` in the aforementioned `CoeOut` instance, for example) happening here which is rather convenient, but it's possible it may cause problems. (this abuse was also present in mathlib3)
3. What should the name of this file be? `LpSpace` seems wrong semantically, but `lpSpace` doesn't seem allowable by our file name conventions.



Co-authored-by: Ruben Van de Velde <65514131+Ruben-VandeVelde@users.noreply.github.com>
Co-authored-by: Moritz Firsching <firsching@google.com>
Co-authored-by: Jireh Loreaux <loreaujy@gmail.com>
  • Loading branch information
4 people committed Jun 1, 2023
1 parent 785b825 commit bc20bc9
Show file tree
Hide file tree
Showing 2 changed files with 1,220 additions and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -552,6 +552,7 @@ import Mathlib.Analysis.NormedSpace.IndicatorFunction
import Mathlib.Analysis.NormedSpace.Int
import Mathlib.Analysis.NormedSpace.IsROrC
import Mathlib.Analysis.NormedSpace.LinearIsometry
import Mathlib.Analysis.NormedSpace.LpSpace
import Mathlib.Analysis.NormedSpace.MStructure
import Mathlib.Analysis.NormedSpace.MazurUlam
import Mathlib.Analysis.NormedSpace.Multilinear
Expand Down

0 comments on commit bc20bc9

Please sign in to comment.