Skip to content

Conversation

fbarroero
Copy link
Collaborator

@fbarroero fbarroero commented Oct 14, 2025

We prove
theorem logMahlerMeasure_X_sub_C (z : ℂ) : (X - C z).logMahlerMeasure = log⁺ ‖z‖
and
theorem logMahlerMeasure_eq_log_leadingCoeff_add_sum_log_roots (p : ℂ[X]) : p.logMahlerMeasure = log ‖p.leadingCoeff‖ + ((p.roots).map (fun a ↦ log⁺ ‖a‖)).sum


Open in Gitpod

@github-actions github-actions bot added t-analysis Analysis (normed *, calculus) large-import Automatically added label for PRs with a significant increase in transitive imports labels Oct 14, 2025
@fbarroero fbarroero added the WIP Work in progress label Oct 14, 2025
@github-actions
Copy link

github-actions bot commented Oct 14, 2025

PR summary 71a105d772

Import changes exceeding 2%

% File
+6.94% Mathlib.Analysis.Polynomial.MahlerMeasure

Import changes for modified files

Dependency changes

File Base Count Head Count Change
Mathlib.Analysis.Polynomial.MahlerMeasure 2480 2652 +172 (+6.94%)
Import changes for all files
Files Import difference
Mathlib.Analysis.Polynomial.MahlerMeasure 172

Declarations diff

+ logMahlerMeasure_C_mul
+ logMahlerMeasure_C_mul_X_add_C
+ logMahlerMeasure_X_add_C
+ logMahlerMeasure_X_sub_C
+ logMahlerMeasure_degree_eq_one
+ logMahlerMeasure_eq_log_leadingCoeff_add_sum_log_roots
+ mahlerMeasure_C_mul_X_add_C
+ mahlerMeasure_X_add_C
+ mahlerMeasure_X_sub_C
+ mahlerMeasure_degree_eq_one
+ mahlerMeasure_eq_leadingCoeff_mul_prod_roots

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).

@fbarroero fbarroero removed the WIP Work in progress label Oct 14, 2025
@fbarroero fbarroero added the WIP Work in progress label Oct 19, 2025
@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 Oct 19, 2025
@mathlib4-merge-conflict-bot mathlib4-merge-conflict-bot added the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Oct 22, 2025
@mathlib4-merge-conflict-bot
Copy link
Collaborator

This pull request has conflicts, please merge master and resolve them.

@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot removed the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label Oct 22, 2025
@mathlib4-dependent-issues-bot
Copy link
Collaborator

@mathlib4-merge-conflict-bot mathlib4-merge-conflict-bot removed the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Oct 22, 2025
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

large-import Automatically added label for PRs with a significant increase in transitive imports t-analysis Analysis (normed *, calculus) WIP Work in progress

Projects

None yet

Development

Successfully merging this pull request may close these issues.

3 participants