mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat: bounds for modular forms of non-positive weights

Open CBirkbeck opened this issue 1 year ago • 1 comments

We use the Maximum modulus principle to show that modular forms of non-positive weights are bounded by its value of some element of the upper half plane imaginary part at least 1/2.


Open in Gitpod

CBirkbeck avatar Oct 24 '24 17:10 CBirkbeck

PR summary 7d5154c184

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.NumberTheory.ModularForms.LevelOne 1646

Declarations diff

+ SlashInvariantForm.exists_one_half_le_im_and_norm_le + SlashInvariantForm.wt_eq_zero_of_eq_const + coe + coe_apply_complex + denom_S + denom_one + det_coe + exists_one_half_le_im_smul + exists_one_half_le_im_smul_and_norm_denom_le + three_le_four_mul_im_sq_of_mem_fd -++- im_smul_eq_div_normSq

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.


Decrease in tech debt: (relative, absolute) = (1.00, 0.00)
Current number Change Type
1552 -1 erw

Current commit 7d5154c184 Reference commit 66df24a8e2

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 Oct 24 '24 17:10 github-actions[bot]

Following some discussion with @CBirkbeck, I've pushed some changes to this branch which avoid making subgroups of SL2Z into subtypes, which gets rid of some unnecessary coercions and API lemmas.

loefflerd avatar Oct 28 '24 18:10 loefflerd

⚠️ The sha of the head commit of this PR conflicts with #18385. Mergify cannot evaluate rules on this PR. ⚠️

mergify[bot] avatar Oct 29 '24 13:10 mergify[bot]

I made #18385 to make the reviewing easier. That PR contains all the q.o.l improvements, this has the new results.

CBirkbeck avatar Oct 29 '24 13:10 CBirkbeck

This PR/issue depends on:

  • ~~leanprover-community/mathlib4#18385~~ By Dependent Issues (🤖). Happy coding!

This had a merge-conflict because of #18385. I merged it with the latest master and sorted out the conflicts, ready for review again.

loefflerd avatar Nov 10 '24 14:11 loefflerd

This had a merge-conflict because of #18385. I merged it with the latest master and sorted out the conflicts, ready for review again.

thanks for doing this and again below!

CBirkbeck avatar Nov 18 '24 10:11 CBirkbeck

No problem! By the way, I realised while fixing the conflicts that we have two distinct namespaces ModularGroup and UpperHalfPlane.ModularGroup. Is this deliberate or should they be unified? In any case denom_one as presently formulated shouldn't be in the ModularGroup namespace, since the 1 is getting elaborated as 1 : ↥GL(2, ℝ)⁺ rather than as 1 : SL(2, ℤ).

loefflerd avatar Nov 18 '24 10:11 loefflerd

No problem! By the way, I realised while fixing the conflicts that we have two distinct namespaces ModularGroup and UpperHalfPlane.ModularGroup. Is this deliberate or should they be unified? In any case denom_one as presently formulated shouldn't be in the ModularGroup namespace, since the 1 is getting elaborated as 1 : ↥GL(2, ℝ)⁺ rather than as 1 : SL(2, ℤ).

No that was a mistake. I've removed it now and move denom_one.

CBirkbeck avatar Nov 19 '24 09:11 CBirkbeck

(I can push fixes with all these changes to your PR, just let me know if that's OK with you.)

loefflerd avatar Nov 19 '24 18:11 loefflerd

(I can push fixes with all these changes to your PR, just let me know if that's OK with you.)

Oh I was just doing this now. Go ahead and I'll double check there is nothing missing.

CBirkbeck avatar Nov 19 '24 18:11 CBirkbeck

I have pushed fixes, I believe everything outside the new file LevelOne is now OK. I have not looked in detail at the new file, other than fixing knock-on effects of the changes I made elsewhere. Looking at it now.

loefflerd avatar Nov 19 '24 18:11 loefflerd

I think the results like modular_S_smul and those near it should maybe also move down

That doesn't work because it's used in exists_SL2_smul_eq_of_apply_zero_one_ne_zero (which is definitely not a ModularGroup lemma).

loefflerd avatar Nov 19 '24 18:11 loefflerd

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

github-actions[bot] avatar Nov 20 '24 08:11 github-actions[bot]

Thanks!

bors d+

riccardobrasca avatar Nov 20 '24 08:11 riccardobrasca

:v: CBirkbeck 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 Nov 20 '24 08:11 mathlib-bors[bot]

bors r+

CBirkbeck avatar Nov 20 '24 10:11 CBirkbeck

Pull request successfully merged into master.

Build succeeded:

mathlib-bors[bot] avatar Nov 20 '24 10:11 mathlib-bors[bot]