Skip to content

Conversation

@github-actions
Copy link

github-actions bot commented Jan 6, 2026

PR summary cb3ccde1ed

Import changes for modified files

Dependency changes

File Base Count Head Count Change
Mathlib.LinearAlgebra.Transvection 1408 0 -1408 (-100.00%)
Import changes for all files
Files Import difference
Mathlib.LinearAlgebra.Transvection -1408
Mathlib.LinearAlgebra.Transvection.Basic (new file) 1425
Mathlib.LinearAlgebra.Center (new file) 1426
Mathlib.LinearAlgebra.Transvection.Generation (new file) 1427
Mathlib.LinearAlgebra.Transvection.SpecialLinearGroup (new file) 1429

Declarations diff

+ Finset.iInf_univ
+ IsBaseChange.transvection
+ IsExceptional
+ IsExceptional.notMem_transvections_pow
+ LinearEquiv.transvection.baseChange
+ LinearIndependent.pair_smul_smul_iff
+ LinearMap.transvection.baseChange
+ _root_.LinearEquiv.det_fixedReduce
+ _root_.LinearEquiv.transvection.det_eq_one
+ _root_.Module.Free.of_det_ne_one
+ closure_pow_le
+ coe_restrict
+ commute_transvections_iff_of_basis
+ comp_smul_smul
+ det
+ det_ofDomain
+ det_ofField
+ dilatransvection
+ dilatransvection.apply
+ dilatransvection.coe_toLinearMap
+ dilatransvection_mem_dilatransvections
+ dilatransvections
+ dilatransvections_pow_mono
+ eq_top_iff_finrank_eq
+ exists_basis_of_pairing_eq_zero
+ exists_basis_of_pairing_ne_zero
+ exists_eq_smul_id_of_forall_notLinearIndependent
+ exists_mem_center_apply_eq_smul_of_forall_notLinearIndependent
+ exists_mem_center_apply_eq_smul_of_forall_notLinearIndependent_of_basis
+ finrank_fixedSubmodule_add_le
+ finrank_fixedSubmodule_dilatransvection_mul_le
+ finrank_fixedSubmodule_mul_dilatransvection_le
+ finrank_le_one_add_finrank_fixedSubmodule_dilatransvection
+ finrank_quotient_fixedSubmodule_of_mem_dilatransvections_pow
+ finrank_quotient_iInf_le_sum_finrank_quotient
+ finrank_quotient_inf_le_finrank_quotient_add_finrank_quotient
+ finrank_quotient_inf_le_finrank_quotient_add_finrank_quotient'
+ finrank_sup_span_singleton
+ fixedReduce_eq_one
+ fixedReduce_eq_smul_iff
+ fixedReduce_mem_dilatransvections_pow
+ fixedReduce_mem_transvections_mul_dilatransvections_pow
+ fixedReduce_mem_transvections_pow_mul_dilatransvections
+ fixedReduce_mk
+ fixedReduce_mkQ
+ fixedSubmodule
+ fixedSubmodule_eq_ker
+ fixedSubmodule_eq_top_iff
+ fixedSubmodule_mul_inf_fixedSubmodule_le_fixedSubmodule
+ fixedSubmodule_mul_inf_fixedSubmodule_le_fixedSubmodule'
+ fixedSubmodule_transvection_mul
+ fixingSubgroup_le_stabilizer
+ iInf_fixedSubmodule_le_fixedSubmodule_prod
+ inf_fixedSubmodule_le_fixedSubmodule_mul
+ inv_mem_dilatransvections_iff
+ ker_le_fixedSubmodule_transvection
+ le_one_add_finrank_fixedSubmodule_dilatransvection_mul
+ le_one_add_finrank_fixedSubmodule_dilatransvection_mul'
+ le_one_add_finrank_fixedSubmodule_mul_dilatransvection
+ map_eq_of_mem_fixingSubgroup
+ mem_center_of_apply_eq_smul
+ mem_dilatransvections_iff_finrank
+ mem_dilatransvections_iff_finrank_quotient
+ mem_dilatransvections_iff_rank
+ mem_dilatransvections_iff_rank_quotient
+ mem_dilatransvections_pow
+ mem_fixedSubmodule_iff
+ mem_fixedSubmodule_transvection_iff
+ mem_stabilizer_fixedSubmodule
+ mem_stabilizer_submodule
+ mem_stabilizer_submodule_iff_map_eq
+ mem_stabilizer_submodule_of_le_fixedSubmodule
+ mem_transvections_iff'
+ mem_transvections_iff_coe
+ mem_transvections_pow
+ mem_transvections_pow_mul_dilatransvections
+ mem_transvections_pow_mul_dilatransvections_of_fixedReduce_eq_one
+ mem_transvections_pow_mul_dilatransvections_of_fixedReduce_ne_smul_id
+ mem_transvections_pow_mul_dilatransvections_of_notIsExceptional
+ mem_transvections_pow_of_notIsExceptional
+ mem_transvections_pow_of_toLinearEquiv
+ notIsExceptional_of_mem_transvections_mul_dilatransvections_pow
+ notIsExceptional_of_mem_transvections_pow_mul_dilatransvections
+ notMem_transvections_mul_dilatransvections_pow
+ one_mem_dilatransvections
+ reduce
+ reduce_mem_dilatransvections
+ reduce_mem_transvections
+ reduce_mk
+ reduce_mkQ
+ restrict
+ smul_submodule_def
+ sup_span_eq_top
+ symm_apply
+ transvection
+ transvection.coe_toLinearEquiv
+ transvection_mem_dilatransvections
+ transvection_mem_transvections
+ transvections_subset_dilatransvections
++ fixedReduce
++ inv_mem_transvections_iff
++ mem_transvections
++ mem_transvections_iff
++ one_mem_transvections
++ subgroup_closure_dilatransvections_eq_top
++ transvections
++ transvections_pow_mono
- _root_.IsBaseChange.transvection
- _root_.LinearEquiv.transvection.baseChange
- baseChange

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

note: file Mathlib/LinearAlgebra/Transvection.lean was removed.
Please create a follow-up pull request adding a module deprecation. Thanks!

@github-actions github-actions bot added the t-algebra Algebra (groups, rings, fields, etc) label Jan 6, 2026
@github-actions github-actions bot added the file-removed A Lean module was (re)moved without a `deprecated_module` annotation label Jan 7, 2026
@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 7, 2026
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) file-removed A Lean module was (re)moved without a `deprecated_module` annotation t-algebra Algebra (groups, rings, fields, etc)

Projects

None yet

Development

Successfully merging this pull request may close these issues.

2 participants