Skip to content

Conversation

@mans0954
Copy link
Collaborator

@mans0954 mans0954 commented Nov 3, 2024

Three lemmas about Quadratic maps applied to:

  • A finite sum
  • A linearCombination
  • The representation of an element wrt a basis

Open in Gitpod

@mans0954 mans0954 added the t-algebra Algebra (groups, rings, fields, etc) label Nov 3, 2024
@github-actions
Copy link

github-actions bot commented Nov 3, 2024

PR summary b7c0de9e62

Import changes for modified files

Dependency changes

File Base Count Head Count Change
Mathlib.LinearAlgebra.QuadraticForm.Basis 1470 1472 +2 (+0.14%)
Import changes for all files
Files Import difference
Mathlib.LinearAlgebra.QuadraticForm.Basis 2
Mathlib.Data.Sym.Sym2.Finsupp (new file) 553

Declarations diff

+ apply_linearCombination
+ apply_linearCombination'
+ coe_sym2Mul
+ map_finsuppSum
+ map_finsuppSum'
+ mem_sym2_support_of_mul_ne_zero
+ polarSym2_map_smul
+ sum_polar_sub_repr_sq
+ sum_repr_sq_add_sum_repr_mul_polar
+ support_sym2Mul_subset
+ sym2Mul
+ sym2Mul_apply_mk
+ sym2_support_eq_preimage_support_mul

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

@mans0954 mans0954 marked this pull request as ready for review November 3, 2024 14:43
@mans0954 mans0954 requested a review from eric-wieser November 3, 2024 14:43
@mans0954
Copy link
Collaborator Author

mans0954 commented Nov 3, 2024

CC: @eric-wieser

@mans0954 mans0954 added the WIP Work in progress label Nov 5, 2024
@mans0954 mans0954 removed the request for review from eric-wieser November 6, 2024 08:22
@mans0954 mans0954 marked this pull request as draft November 6, 2024 08:23
@mans0954 mans0954 marked this pull request as ready for review November 6, 2024 18:03
@mans0954 mans0954 removed the WIP Work in progress label Nov 6, 2024
@Ruben-VandeVelde Ruben-VandeVelde changed the title feature(LinearAlgebra/QuadraticForm/Basis): basis expansion of a quadratic map feat(LinearAlgebra/QuadraticForm/Basis): basis expansion of a quadratic map Nov 6, 2024
mans0954 added a commit that referenced this pull request Nov 24, 2024
@YaelDillies YaelDillies added awaiting-author A reviewer has asked the author a question or requested changes. and removed maintainer-merge A reviewer has approved the changed; awaiting maintainer approval. labels Apr 5, 2025
@mans0954 mans0954 removed the awaiting-author A reviewer has asked the author a question or requested changes. label Apr 5, 2025
Copy link
Collaborator

@YaelDillies YaelDillies left a comment

Choose a reason for hiding this comment

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

Let's try again

maintainer merge

@github-actions
Copy link

github-actions bot commented Apr 5, 2025

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

@github-actions github-actions bot added the maintainer-merge A reviewer has approved the changed; awaiting maintainer approval. label Apr 5, 2025
@riccardobrasca
Copy link
Member

This went through an insane amount of review, so let's just merge it, thanks!

bors merge

@leanprover-community-mathlib4-bot leanprover-community-mathlib4-bot added ready-to-merge This PR has been sent to bors. and removed maintainer-merge A reviewer has approved the changed; awaiting maintainer approval. labels Apr 6, 2025
mathlib-bors bot pushed a commit that referenced this pull request Apr 6, 2025
…ic map (#18578)

Three lemmas about Quadratic maps applied to:

- A finite sum
- A `linearCombination`
- The representation of an element wrt a basis



Co-authored-by: Christopher Hoskin <christopher.hoskin@gmail.com>
Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Apr 6, 2025

Build failed (retrying...):

mathlib-bors bot pushed a commit that referenced this pull request Apr 6, 2025
…ic map (#18578)

Three lemmas about Quadratic maps applied to:

- A finite sum
- A `linearCombination`
- The representation of an element wrt a basis



Co-authored-by: Christopher Hoskin <christopher.hoskin@gmail.com>
Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Apr 6, 2025

Build failed (retrying...):

mathlib-bors bot pushed a commit that referenced this pull request Apr 6, 2025
…ic map (#18578)

Three lemmas about Quadratic maps applied to:

- A finite sum
- A `linearCombination`
- The representation of an element wrt a basis



Co-authored-by: Christopher Hoskin <christopher.hoskin@gmail.com>
Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Apr 6, 2025

Build failed:

@eric-wieser
Copy link
Member

bors merge

mathlib-bors bot pushed a commit that referenced this pull request Apr 6, 2025
…ic map (#18578)

Three lemmas about Quadratic maps applied to:

- A finite sum
- A `linearCombination`
- The representation of an element wrt a basis



Co-authored-by: Christopher Hoskin <mans0954@users.noreply.github.com>
Co-authored-by: Christopher Hoskin <christopher.hoskin@gmail.com>
Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
@mathlib-bors
Copy link
Contributor

mathlib-bors bot commented Apr 6, 2025

Pull request successfully merged into master.

Build succeeded:

@mathlib-bors mathlib-bors bot changed the title feat(LinearAlgebra/QuadraticForm/Basis): basis expansion of a quadratic map [Merged by Bors] - feat(LinearAlgebra/QuadraticForm/Basis): basis expansion of a quadratic map Apr 6, 2025
@mathlib-bors mathlib-bors bot closed this Apr 6, 2025
@mathlib-bors mathlib-bors bot deleted the mans0954/quadratic-basis_expansion branch April 6, 2025 22:28
tannerduve pushed a commit that referenced this pull request May 13, 2025
…ic map (#18578)

Three lemmas about Quadratic maps applied to:

- A finite sum
- A `linearCombination`
- The representation of an element wrt a basis



Co-authored-by: Christopher Hoskin <mans0954@users.noreply.github.com>
Co-authored-by: Christopher Hoskin <christopher.hoskin@gmail.com>
Co-authored-by: Yaël Dillies <yael.dillies@gmail.com>
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

ready-to-merge This PR has been sent to bors. t-algebra Algebra (groups, rings, fields, etc)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

9 participants