Skip to content

Conversation

@sgouezel
Copy link
Contributor

Zulip discussion at #mathlib4 > Duplication @ 💬


Open in Gitpod

@github-actions github-actions bot added the t-analysis Analysis (normed *, calculus) label Dec 26, 2025
@github-actions
Copy link

github-actions bot commented Dec 26, 2025

PR summary 0bf098cae7

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ orthogonalBilin_innerₗ

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

LinearMap.mk₂'ₛₗ (RingHom.id 𝕜) (starRingEnd _) (fun x y => ⟪y, x⟫)
(fun _x _y _z => inner_add_right _ _ _) (fun _r _x _y => inner_smul_right _ _ _)
(fun _x _y _z => inner_add_left _ _ _) fun _r _x _y => inner_smul_left _ _ _
def innerₛₗ : E →ₗ⋆[𝕜] E →ₗ[𝕜] 𝕜 :=
Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Getting rid of the duplication is fine, but the other name comes off as more readable to me. I thought using non-ASCII characters in declarations was generally discouraged.

Copy link
Contributor Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

innerₛₗ is the standard spelling throughout mathlib (used 10 times more than the other one). This PR is only about removing the duplication, not changing the name. This could be done later in another PR if needed, but I think a prerequisite would be to converge on a naming scheme for our whole zoo of bundled linear maps, bilinear maps, continuous linear maps and so on.

Copy link
Member

@jcommelin jcommelin left a comment

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Thanks 🎉

bors d+

@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Dec 27, 2025

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

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the delegated This pull request has been delegated to the PR author (or occasionally another non-maintainer). label Dec 27, 2025
sgouezel and others added 3 commits December 27, 2025 10:39
Co-authored-by: Moritz Doll <moritz.doll@googlemail.com>
Co-authored-by: Moritz Doll <moritz.doll@googlemail.com>
Co-authored-by: Moritz Doll <moritz.doll@googlemail.com>
@sgouezel
Copy link
Contributor Author

bors r+

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added the ready-to-merge This PR has been sent to bors. label Dec 27, 2025
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Dec 27, 2025

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title chore: deprecate duplicate declaration for the scalar product as a sesquilinear form [Merged by Bors] - chore: deprecate duplicate declaration for the scalar product as a sesquilinear form Dec 27, 2025
@mathlib-bors mathlib-bors bot closed this Dec 27, 2025
kim-em pushed a commit to kim-em/mathlib4 that referenced this pull request Jan 6, 2026
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

delegated This pull request has been delegated to the PR author (or occasionally another non-maintainer). ready-to-merge This PR has been sent to bors. t-analysis Analysis (normed *, calculus)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

5 participants