Skip to content

Conversation

@jonwashburn
Copy link

PR 3c on HadamardFactorization pipeline
Co-authored with Matteo Cipollina (matteo.cipollina@yahoo.it)


Open in Gitpod

@github-actions github-actions bot added new-contributor This PR was made by a contributor with at most 5 merged PRs. Welcome to the community! t-analysis Analysis (normed *, calculus) labels Jan 23, 2026
@github-actions
Copy link

PR summary 18ef4ef4f3

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.Analysis.SpecialFunctions.Gamma.BinetKernel (new file) 2495

Declarations diff

+ K
+ K_eq_alt
+ K_eq_alt'
+ K_nonneg
+ K_pos
+ Ktilde
+ Ktilde_bdd
+ Ktilde_ge_one_div_twelve_mul_exp_neg_div_twelve
+ Ktilde_le
+ Ktilde_lt
+ Ktilde_nonneg
+ Ktilde_pos
+ Ktilde_zero
+ continuousOn_Ktilde_Ioi
+ continuous_Ktilde
+ differentiableOn_gAux
+ differentiableOn_gAux'
+ differentiableOn_gAux''
+ differentiableOn_robbinsAux
+ differentiableOn_robbinsAux'
+ differentiableOn_robbinsAux''
+ differentiableOn_robbinsAux'''
+ exp_mul_one_sub_lt_one
+ exp_sub_one_pos
+ f
+ f_at_one
+ f_deriv
+ f_deriv'
+ f_deriv_pos
+ f_nonneg
+ f_one_pos
+ f_zero
+ gAux
+ gAux'
+ gAux''
+ gAux'''
+ gAux'''_nonneg
+ gAux'''_pos
+ gAux''_nonneg
+ gAux''_pos
+ gAux''_zero
+ gAux'_nonneg
+ gAux'_pos
+ gAux'_zero
+ gAux_nonneg
+ gAux_pos
+ gAux_zero
+ hasDerivAt_gAux
+ hasDerivAt_gAux'
+ hasDerivAt_gAux''
+ hasDerivAt_robbinsAux
+ hasDerivAt_robbinsAux'
+ hasDerivAt_robbinsAux''
+ hasDerivAt_robbinsAux'''
+ hasDerivAt_robbinsPoly
+ integrable_Ktilde_exp
+ integrable_Ktilde_exp_complex
+ monotoneOn_of_deriv_nonneg_Ici
+ nonneg_of_deriv_nonneg_Ici
+ robbinsAux
+ robbinsAux'
+ robbinsAux''
+ robbinsAux'''
+ robbinsAux''''
+ robbinsAux''''_nonneg
+ robbinsAux'''_nonneg
+ robbinsAux'''_zero
+ robbinsAux''_nonneg
+ robbinsAux''_zero
+ robbinsAux'_nonneg
+ robbinsAux'_zero
+ robbinsAux_nonneg
+ robbinsAux_zero
+ robbinsPoly
+ robbinsPoly'
+ robbinsPoly'_pos
+ robbinsPoly_pos
+ tendsto_Ktilde_zero
+ tendsto_exp_sub_one_div
+ tendsto_exp_taylor3_div_cube
+ tendsto_f_div_cube

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
Copy link

🚨 PR Title Needs Formatting

Please update the title to match our commit style conventions.

Errors from script:

error: the PR title should be of the form
  abbrev: main title
or
  abbrev(scope): main title
Details on the required title format

The title should fit the following format:

<kind>(<optional-scope>): <subject>

<kind> is:

  • feat (feature)
  • fix (bug fix)
  • doc (documentation)
  • style (formatting, missing semicolons, ...)
  • refactor
  • test (when adding missing tests)
  • chore (maintain)
  • perf (performance improvement, optimization, ...)
  • ci (changes to continuous integration, repo automation, ...)

<optional-scope> is a name of module or a directory which contains changed modules.
This is not necessary to include, but may be useful if the <subject> is insufficient.
The Mathlib directory prefix is always omitted.
For instance, it could be

  • Data/Nat/Basic
  • Algebra/Group/Defs
  • Topology/Constructions

<subject> has the following constraints:

  • do not capitalize the first letter
  • no dot(.) at the end
  • use imperative, present tense: "change" not "changed" nor "changes"

@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot added the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label Jan 23, 2026
@mathlib4-dependent-issues-bot
Copy link
Collaborator

This PR/issue depends on:

Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) new-contributor This PR was made by a contributor with at most 5 merged PRs. Welcome to the community! t-analysis Analysis (normed *, calculus)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

4 participants