mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat(Analysis.Normed.Ring.Seminorm): add SmoothingSeminorm

Open mariainesdff opened this issue 1 year ago • 3 comments

We prove [BGR, Proposition 1.3.2/1][bosch-guntzer-remmert] : if f is a nonarchimedean seminorm on R, then iInf (λ (n : pnat), (f(x^(n : ℕ)))^(1/(n : ℝ))) is a power-multiplicative nonarchimedean seminorm on R.


  • [ ] depends on: #18173
  • [ ] depends on: #18172
  • [ ] depends on: #18171
  • [x] depends on: #16767
  • [x] depends on: #16768
  • [x] depends on: #16770

Open in Gitpod

mariainesdff avatar Jul 31 '24 16:07 mariainesdff

PR summary e1af4db594

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.Analysis.Normed.Ring.SmoothingSeminorm (new file) 1603

Declarations diff

+ isNonarchimedean_smoothingFun + isPowMul_smoothingFun + pow_mul_apply_eq_pow_mul + smoothingFun + smoothingFun_apply_of_map_mul_eq_mul + smoothingFun_le + smoothingFun_le_self + smoothingFun_nonneg + smoothingFun_of_map_mul_eq_mul + smoothingFun_of_powMul + smoothingFun_one_le + smoothingSeminorm + smoothingSeminormSeq + smoothingSeminormSeq_bddBelow + smoothingSeminorm_apply_of_map_mul_eq_mul + smoothingSeminorm_map_one_le_one + smoothingSeminorm_of_mul + tendsto_smoothingFun_comp + tendsto_smoothingFun_of_eq_zero + tendsto_smoothingFun_of_map_one_le_one + tendsto_smoothingFun_of_ne_zero + zero_mem_lowerBounds_smoothingSeminormSeq_range

You can run this locally as follows
## summary with just the declaration names:
./scripts/declarations_diff.sh <optional_commit>

## more verbose report:
./scripts/declarations_diff.sh long <optional_commit>

The doc-module for script/declarations_diff.sh contains some details about this script.


No changes to technical debt.

You can run this locally as

./scripts/technical-debt-metrics.sh pr_summary
  • The relative value is the weighted sum of the differences with weight given by the inverse of the current value of the statistic.
  • The absolute value is the relative value divided by the total sum of the inverses of the current values (i.e. the weighted average of the differences).

github-actions[bot] avatar Jul 31 '24 16:07 github-actions[bot]

This PR is quite large. Are you planning to split it up?

jcommelin avatar Sep 12 '24 07:09 jcommelin

This PR/issue depends on:

  • ~~leanprover-community/mathlib4#18173~~
  • ~~leanprover-community/mathlib4#18172~~
  • ~~leanprover-community/mathlib4#18171~~
  • ~~leanprover-community/mathlib4#16767~~
  • ~~leanprover-community/mathlib4#16768~~
  • ~~leanprover-community/mathlib4#16770~~ By Dependent Issues (🤖). Happy coding!

Haven't looked at the mathematics, but here's style and naming comments

Thanks!

mariainesdff avatar Jan 17 '25 11:01 mariainesdff

I left some answers to your comments, I'll now check the remaining sections.

faenuccio avatar Jan 28 '25 15:01 faenuccio

Thanks for all the work, LGTM!

faenuccio avatar Feb 05 '25 18:02 faenuccio

maintainer merge

faenuccio avatar Feb 05 '25 18:02 faenuccio

🚀 Pull request has been placed on the maintainer queue by faenuccio.

github-actions[bot] avatar Feb 05 '25 18:02 github-actions[bot]

:v: mariainesdff can now approve this pull request. To approve and merge a pull request, simply reply with bors r+. More detailed instructions are available here.

mathlib-bors[bot] avatar Feb 07 '25 07:02 mathlib-bors[bot]

Build failed (retrying...):

mathlib-bors[bot] avatar Feb 07 '25 18:02 mathlib-bors[bot]

bors r-

Please merge master, fix the build and place back on the queue by commenting bors merge. Thanks!

bryangingechen avatar Feb 07 '25 18:02 bryangingechen

Canceled.

mathlib-bors[bot] avatar Feb 07 '25 18:02 mathlib-bors[bot]

bors r+

mariainesdff avatar Feb 10 '25 10:02 mariainesdff

Pull request successfully merged into master.

Build succeeded:

mathlib-bors[bot] avatar Feb 10 '25 13:02 mathlib-bors[bot]