Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

feat(number_theory/bernoulli): simplify bernoulli power series #6641

Closed
wants to merge 3 commits into from

Conversation

mo271
Copy link
Collaborator

@mo271 mo271 commented Mar 11, 2021

Now using exp_bernoulli_poly to prove both bernoulli'_power_series_mul_exp_sub_one and
bernoulli_power_series_mul_exp_sub_one


@mo271 mo271 marked this pull request as draft March 11, 2021 14:30
@mo271
Copy link
Collaborator Author

mo271 commented Mar 11, 2021

This change was suggest here: #6309 (comment).
Currently two thing need to be done:

  • Avoid circular imports: I moved bernoulli'_power_series_mul_exp_sub_one,
    bernoulli_power_series_mul_exp_sub_one, bernoulli_power_series and bernoulli'_power_series to the file bernoulli_polynomial.lean. This results in problems in the file bernoulli.lean because bernoulli'_odd_eq_zero uses bernoulli'_power_series_mul_exp_sub_one. How to resolve that best?
    I guess one way would be to put bernoulli'_odd_eq_zero and everthing that depends on it to bernoulli_polynomial, but maybe there are better ways,
  • There are two lemmas that seem so simple that I would have expected that they exists already, and I simply didn't find them.
    (on going discussion here: https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there.20code.20for.20X.3F/topic/poly.20(a)eval.20and.20algebra.20maps )

@github-actions github-actions bot added the blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. label Mar 11, 2021
@mo271 mo271 added the help-wanted The author needs attention to resolve issues label Mar 11, 2021
@mo271
Copy link
Collaborator Author

mo271 commented Mar 11, 2021

help wanted for the question above about where to put this best in order to avoid circular dependencies!

@github-actions github-actions bot removed the blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. label Mar 14, 2021
@github-actions
Copy link

🎉 Great news! Looks like all the dependencies have been resolved:

💡 To add or remove a dependency please update this issue/PR description.

Brought to you by Dependent Issues (:robot: ). Happy coding!

@mo271
Copy link
Collaborator Author

mo271 commented Mar 14, 2021

I looked at this again and was surprised that bernoulli_odd_eq_zero uses bernoulli'_power_series_mul_exp_sub_one. Unfortunately, this leads to a circular dependence like this where each line depends on the one before:

  • sum_bernoulli
  • bernoulli_eq_bernoulli'_of_ne_one
  • bernoulli_odd_eq_zero
  • bernoulli'_power_series_mul_exp_sub_one
  • exp_bernoulli_poly
  • sum_bernoulli_poly
  • sum_bernoulli
    This means that unless we come up with a way to break this chain somehow, we should stick with the longer proof that we currently have for bernoulli'_power_series_mul_exp_sub_one.

@mo271 mo271 closed this Mar 14, 2021
@YaelDillies YaelDillies deleted the new_bernoulli_power_series branch June 11, 2023 17:22
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
help-wanted The author needs attention to resolve issues
Projects
None yet
Development

Successfully merging this pull request may close these issues.

2 participants