Skip to content

Commit 12ba7ac

Browse files
author
mathlib4-bot
committed
Auto-resolved conflicts in lean-toolchain and lake-manifest.json
2 parents f0b00a6 + 7d5bdba commit 12ba7ac

File tree

94 files changed

+2869
-989
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

94 files changed

+2869
-989
lines changed

.github/workflows/PR_summary.yml

Lines changed: 23 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -13,9 +13,19 @@ jobs:
1313
uses: actions/checkout@11bd71901bbe5b1630ceea73d27597364c9af683 # v4.2.2
1414
with:
1515
fetch-depth: 0
16+
path: pr-branch
17+
18+
# Checkout the master branch into a subdirectory
19+
- name: Checkout master branch
20+
uses: actions/checkout@11bd71901bbe5b1630ceea73d27597364c9af683 # v4.2.2
21+
with:
22+
# When testing the scripts, comment out the "ref: master"
23+
ref: master
24+
path: master-branch
1625

1726
- name: Update the merge-conflict label
1827
run: |
28+
cd pr-branch
1929
printf 'PR number: "%s"\n' "${{ github.event.pull_request.number }}"
2030
if git merge origin/master --no-ff --no-commit
2131
then
@@ -27,7 +37,7 @@ jobs:
2737
--url https://api.github.com/repos/${{ github.repository }}/issues/${{ github.event.pull_request.number }}/labels/merge-conflict \
2838
--header 'authorization: Bearer ${{ secrets.GITHUB_TOKEN }}'
2939
else
30-
echo "This PR has merge conflicts with main."
40+
echo "This PR has merge conflicts with master."
3141
# we use curl rather than octokit/request-action so that the job won't fail
3242
# (and send an annoying email) if the labels don't exist
3343
curl --request POST \
@@ -36,7 +46,6 @@ jobs:
3646
--header 'X-GitHub-Api-Version: 2022-11-28' \
3747
--url https://api.github.com/repos/${{ github.repository }}/issues/${{ github.event.pull_request.number }}/labels \
3848
--data '{"labels":["merge-conflict"]}'
39-
4049
fi
4150
4251
- name: Set up Python
@@ -52,6 +61,7 @@ jobs:
5261
5362
- name: Get changed and removed/renamed files
5463
run: |
64+
cd pr-branch
5565
git fetch origin ${{ github.base_ref }} # fetch the base branch
5666
5767
# Get the list of all changed files.
@@ -87,6 +97,7 @@ jobs:
8797
8898
- name: Compute (re)moved files without deprecation
8999
run: |
100+
cd pr-branch
90101
touch moved_without_deprecation.txt
91102
git checkout ${{ github.base_ref }}
92103
while IFS= read -r file
@@ -112,19 +123,20 @@ jobs:
112123
113124
- name: Compute transitive imports
114125
run: |
126+
cd pr-branch
115127
# the checkout dance, to avoid a detached head
116128
git checkout master
117129
git checkout -
118130
currentHash="$(git rev-parse HEAD)"
119131
120132
# Compute the counts for the HEAD of the PR
121-
python ./scripts/count-trans-deps.py "Mathlib/" > head.json
133+
python ../master-branch/scripts/count-trans-deps.py "Mathlib/" > head.json
122134
123135
# Checkout the merge base
124136
git checkout "$(git merge-base master ${{ github.sha }})"
125137
126138
# Compute the counts for the merge base
127-
python ./scripts/count-trans-deps.py "Mathlib/" > base.json
139+
python ../master-branch/scripts/count-trans-deps.py "Mathlib/" > base.json
128140
129141
# switch back to the current branch: the `declarations_diff` script should be here
130142
git checkout "${currentHash}"
@@ -134,15 +146,16 @@ jobs:
134146
GH_TOKEN: ${{ secrets.GITHUB_TOKEN }}
135147
BRANCH_NAME: ${{ github.head_ref }}
136148
run: |
149+
cd pr-branch
137150
PR="${{ github.event.pull_request.number }}"
138151
title="### PR summary"
139152
140-
graphAndHighPercentReports=$(python ./scripts/import-graph-report.py base.json head.json changed_files.txt)
153+
graphAndHighPercentReports=$(python ../master-branch/scripts/import-graph-report.py base.json head.json changed_files.txt)
141154
142155
## Import count comment
143156
importCount=$(
144157
printf '%s\n' "${graphAndHighPercentReports}" | sed '/^Import changes exceeding/Q'
145-
./scripts/import_trans_difference.sh
158+
../master-branch/scripts/import_trans_difference.sh
146159
)
147160
148161
## High percentage imports
@@ -166,7 +179,7 @@ jobs:
166179
fi
167180
168181
## Declarations' diff comment
169-
declDiff=$(./scripts/declarations_diff.sh)
182+
declDiff=$(../master-branch/scripts/declarations_diff.sh)
170183
if [ "$(printf '%s' "${declDiff}" | wc -l)" -gt 15 ]
171184
then
172185
declDiff="$(printf '<details><summary>\n\n%s\n\n</summary>\n\n%s\n\n</details>\n' "#### Declarations diff" "${declDiff}")"
@@ -178,7 +191,7 @@ jobs:
178191
hashURL="https://github.com/${{ github.repository }}/pull/${{ github.event.pull_request.number }}/commits/${currentHash}"
179192
180193
## Technical debt changes
181-
techDebtVar="$(./scripts/technical-debt-metrics.sh pr_summary)"
194+
techDebtVar="$(../master-branch/scripts/technical-debt-metrics.sh pr_summary)"
182195
183196
# store in a file, to avoid "long arguments" error.
184197
printf '%s [%s](%s)%s\n\n%s\n\n---\n\n%s\n\n---\n\n%s\n' "${title}" "$(git rev-parse --short HEAD)" "${hashURL}" "${high_percentages}" "${importCount}" "${declDiff}" "${techDebtVar}" > please_merge_master.md
@@ -191,10 +204,11 @@ jobs:
191204
fi
192205
193206
cat please_merge_master.md
194-
./scripts/update_PR_comment.sh please_merge_master.md "${title}" "${PR}"
207+
../master-branch/scripts/update_PR_comment.sh please_merge_master.md "${title}" "${PR}"
195208
196209
- name: Update the file-removed label
197210
run: |
211+
cd pr-branch
198212
undeprecatedMoves="$(cat moved_without_deprecation.txt)"
199213
if [ -n "$undeprecatedMoves" ]; then
200214
echo "This PR has undeprecated module (re)movals."

.github/workflows/maintainer_merge.yml

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -113,7 +113,8 @@ jobs:
113113
if: ${{ ! steps.merge_or_delegate.outputs.mOrD == '' }}
114114
uses: actions/github-script@60a0d83039c74a4aee543508d2ffcb1c3799cdea # v7.0.1
115115
with:
116-
github-token: ${{secrets.GITHUB_TOKEN}}
116+
# labels added by GITHUB_TOKEN won't trigger the Zulip emoji workflow
117+
github-token: ${{secrets.TRIAGE_TOKEN}}
117118
script: |
118119
const { owner, repo, number: issue_number } = context.issue;
119120
await github.rest.issues.addLabels({ owner, repo, issue_number, labels: ['maintainer-merge'] });

Counterexamples/AharoniKorman.lean

Lines changed: 0 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -67,10 +67,6 @@ aim of reaching a contradiction (as then, no such partition can exist). We may f
6767
we have a contradiction (`no_spinalMap`), and therefore show that no spinal map exists.
6868
-/
6969

70-
#adaptation_note /-- 2025-03-12
71-
We temporarily comment out this file on `nightly-testing`, awaiting fixes for a complex
72-
interaction between `omega`, `aesop`, and asynchronous elaboration.
73-
7470
attribute [aesop norm 10 tactic] Lean.Elab.Tactic.Omega.omegaDefault
7571
attribute [aesop 2 simp] Set.subset_def Finset.subset_iff
7672

@@ -1253,5 +1249,3 @@ theorem aharoni_korman_false :
12531249
rw [Hollom.exists_partition_iff_nonempty_spinalMap hC] at h
12541250
obtain ⟨f⟩ := h
12551251
exact Hollom.no_spinalMap hC f
1256-
1257-
-/

Mathlib.lean

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1608,8 +1608,10 @@ import Mathlib.Analysis.MellinTransform
16081608
import Mathlib.Analysis.Meromorphic.Basic
16091609
import Mathlib.Analysis.Meromorphic.Divisor
16101610
import Mathlib.Analysis.Meromorphic.FactorizedRational
1611+
import Mathlib.Analysis.Meromorphic.IsolatedZeros
16111612
import Mathlib.Analysis.Meromorphic.NormalForm
16121613
import Mathlib.Analysis.Meromorphic.Order
1614+
import Mathlib.Analysis.Meromorphic.TrailingCoefficient
16131615
import Mathlib.Analysis.Normed.Affine.AddTorsor
16141616
import Mathlib.Analysis.Normed.Affine.AddTorsorBases
16151617
import Mathlib.Analysis.Normed.Affine.ContinuousAffineMap
@@ -1706,6 +1708,7 @@ import Mathlib.Analysis.Normed.Unbundled.SeminormFromConst
17061708
import Mathlib.Analysis.Normed.Unbundled.SmoothingSeminorm
17071709
import Mathlib.Analysis.Normed.Unbundled.SpectralNorm
17081710
import Mathlib.Analysis.NormedSpace.Alternating.Basic
1711+
import Mathlib.Analysis.NormedSpace.Alternating.Curry
17091712
import Mathlib.Analysis.NormedSpace.BallAction
17101713
import Mathlib.Analysis.NormedSpace.ConformalLinearMap
17111714
import Mathlib.Analysis.NormedSpace.Connected
@@ -4563,6 +4566,7 @@ import Mathlib.NumberTheory.MulChar.Lemmas
45634566
import Mathlib.NumberTheory.Multiplicity
45644567
import Mathlib.NumberTheory.NumberField.AdeleRing
45654568
import Mathlib.NumberTheory.NumberField.Basic
4569+
import Mathlib.NumberTheory.NumberField.CMField
45664570
import Mathlib.NumberTheory.NumberField.CanonicalEmbedding.Basic
45674571
import Mathlib.NumberTheory.NumberField.CanonicalEmbedding.ConvexBody
45684572
import Mathlib.NumberTheory.NumberField.CanonicalEmbedding.FundamentalCone
@@ -4999,6 +5003,7 @@ import Mathlib.RepresentationTheory.GroupCohomology.Functoriality
49995003
import Mathlib.RepresentationTheory.GroupCohomology.Hilbert90
50005004
import Mathlib.RepresentationTheory.GroupCohomology.LowDegree
50015005
import Mathlib.RepresentationTheory.GroupCohomology.Resolution
5006+
import Mathlib.RepresentationTheory.Induced
50025007
import Mathlib.RepresentationTheory.Invariants
50035008
import Mathlib.RepresentationTheory.Maschke
50045009
import Mathlib.RepresentationTheory.Rep
@@ -6085,8 +6090,10 @@ import Mathlib.Topology.Closure
60856090
import Mathlib.Topology.ClusterPt
60866091
import Mathlib.Topology.Coherent
60876092
import Mathlib.Topology.CompactOpen
6093+
import Mathlib.Topology.Compactification.OnePoint
60886094
import Mathlib.Topology.Compactification.OnePoint.Basic
60896095
import Mathlib.Topology.Compactification.OnePoint.ProjectiveLine
6096+
import Mathlib.Topology.Compactification.OnePointEquiv
60906097
import Mathlib.Topology.Compactness.Bases
60916098
import Mathlib.Topology.Compactness.Compact
60926099
import Mathlib.Topology.Compactness.CompactlyCoherentSpace

Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean

Lines changed: 27 additions & 25 deletions
Original file line numberDiff line numberDiff line change
@@ -36,18 +36,21 @@ universe v u
3636

3737
namespace CoalgCat
3838

39-
open CategoryTheory MonoidalCategory
39+
open CategoryTheory MonoidalCategory Comon_Class
4040

4141
variable {R : Type u} [CommRing R]
4242

43-
/-- An `R`-coalgebra is a comonoid object in the category of `R`-modules. -/
44-
@[simps X counit comul] def toComonObj (X : CoalgCat R) : Comon_ (ModuleCat R) where
45-
X := ModuleCat.of R X
43+
@[simps counit comul]
44+
noncomputable instance (X : CoalgCat R) : Comon_Class (ModuleCat.of R X) where
4645
counit := ModuleCat.ofHom Coalgebra.counit
4746
comul := ModuleCat.ofHom Coalgebra.comul
48-
counit_comul := ModuleCat.hom_ext <| by simpa using Coalgebra.rTensor_counit_comp_comul
49-
comul_counit := ModuleCat.hom_ext <| by simpa using Coalgebra.lTensor_counit_comp_comul
50-
comul_assoc := ModuleCat.hom_ext <| by simp_rw [ModuleCat.of_coe]; exact Coalgebra.coassoc.symm
47+
counit_comul' := ModuleCat.hom_ext <| by simpa using Coalgebra.rTensor_counit_comp_comul
48+
comul_counit' := ModuleCat.hom_ext <| by simpa using Coalgebra.lTensor_counit_comp_comul
49+
comul_assoc' := ModuleCat.hom_ext <| by simp_rw [ModuleCat.of_coe]; exact Coalgebra.coassoc.symm
50+
51+
/-- An `R`-coalgebra is a comonoid object in the category of `R`-modules. -/
52+
@[simps X]
53+
noncomputable def toComonObj (X : CoalgCat R) : Comon_ (ModuleCat R) := ⟨ModuleCat.of R X⟩
5154

5255
variable (R) in
5356
/-- The natural functor from `R`-coalgebras to comonoid objects in the category of `R`-modules. -/
@@ -62,26 +65,26 @@ def toComon : CoalgCat R ⥤ Comon_ (ModuleCat R) where
6265
/-- A comonoid object in the category of `R`-modules has a natural comultiplication
6366
and counit. -/
6467
@[simps]
65-
noncomputable instance ofComonObjCoalgebraStruct (X : Comon_ (ModuleCat R)) :
66-
CoalgebraStruct R X.X where
67-
comul := X.comul.hom
68-
counit := X.counit.hom
68+
noncomputable instance ofComonObjCoalgebraStruct (X : ModuleCat R) [Comon_Class X] :
69+
CoalgebraStruct R X where
70+
comul := Δ[X].hom
71+
counit := ε[X].hom
6972

7073
/-- A comonoid object in the category of `R`-modules has a natural `R`-coalgebra
7174
structure. -/
72-
def ofComonObj (X : Comon_ (ModuleCat R)) : CoalgCat R :=
73-
{ ModuleCat.of R X.X with
75+
noncomputable def ofComonObj (X : ModuleCat R) [Comon_Class X] : CoalgCat R :=
76+
{ ModuleCat.of R X with
7477
instCoalgebra :=
7578
{ ofComonObjCoalgebraStruct X with
76-
coassoc := ModuleCat.hom_ext_iff.mp X.comul_assoc.symm
77-
rTensor_counit_comp_comul := ModuleCat.hom_ext_iff.mp X.counit_comul
78-
lTensor_counit_comp_comul := ModuleCat.hom_ext_iff.mp X.comul_counit } }
79+
coassoc := ModuleCat.hom_ext_iff.mp (comul_assoc X).symm
80+
rTensor_counit_comp_comul := ModuleCat.hom_ext_iff.mp (counit_comul X)
81+
lTensor_counit_comp_comul := ModuleCat.hom_ext_iff.mp (comul_counit X) } }
7982

8083
variable (R)
8184

8285
/-- The natural functor from comonoid objects in the category of `R`-modules to `R`-coalgebras. -/
83-
def ofComon : Comon_ (ModuleCat R) ⥤ CoalgCat R where
84-
obj X := ofComonObj X
86+
noncomputable def ofComon : Comon_ (ModuleCat R) ⥤ CoalgCat R where
87+
obj X := ofComonObj X.X
8588
map f :=
8689
{ toCoalgHom' :=
8790
{ f.hom.hom with
@@ -122,8 +125,10 @@ theorem tensorObj_comul (K L : CoalgCat R) :
122125
∘ₗ TensorProduct.map Coalgebra.comul Coalgebra.comul := by
123126
rw [ofComonObjCoalgebraStruct_comul]
124127
dsimp only [Equivalence.symm_inverse, comonEquivalence_functor, toComon_obj]
125-
simp only [Comon_.monoidal_tensorObj_comul, toComonObj_X, ModuleCat.of_coe, toComonObj_comul,
126-
tensorμ_eq_tensorTensorTensorComm]
128+
simp only [Comon_.monoidal_tensorObj_comon_comul, Equivalence.symm_inverse,
129+
comonEquivalence_functor, toComon_obj, toComonObj_X, ModuleCat.of_coe, comul_def,
130+
tensorμ_eq_tensorTensorTensorComm, ModuleCat.hom_comp, ModuleCat.hom_ofHom,
131+
LinearEquiv.comp_toLinearMap_eq_iff]
127132
rfl
128133

129134
theorem tensorHom_toLinearMap (f : M →ₗc[R] N) (g : P →ₗc[R] Q) :
@@ -158,9 +163,7 @@ theorem comul_tensorObj_tensorObj_right :
158163
(CoalgCat.of R N ⊗ CoalgCat.of R P) : CoalgCat R))
159164
= Coalgebra.comul (A := M ⊗[R] N ⊗[R] P) := by
160165
rw [ofComonObjCoalgebraStruct_comul]
161-
dsimp
162-
simp only [Comon_.monoidal_tensorObj_comul, toComonObj_comul]
163-
rw [ofComonObjCoalgebraStruct_comul]
166+
simp only [Comon_.monoidal_tensorObj_comon_comul, toComonObj]
164167
simp [tensorμ_eq_tensorTensorTensorComm, TensorProduct.comul_def,
165168
AlgebraTensorModule.tensorTensorTensorComm_eq]
166169
rfl
@@ -171,8 +174,7 @@ theorem comul_tensorObj_tensorObj_left :
171174
= Coalgebra.comul (A := (M ⊗[R] N) ⊗[R] P) := by
172175
rw [ofComonObjCoalgebraStruct_comul]
173176
dsimp
174-
simp only [Comon_.monoidal_tensorObj_comul, toComonObj_comul]
175-
rw [ofComonObjCoalgebraStruct_comul]
177+
simp only [Comon_.monoidal_tensorObj_comon_comul, toComonObj]
176178
simp [tensorμ_eq_tensorTensorTensorComm, TensorProduct.comul_def,
177179
AlgebraTensorModule.tensorTensorTensorComm_eq]
178180
rfl

Mathlib/Algebra/Category/Grp/LeftExactFunctor.lean

Lines changed: 8 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -62,6 +62,8 @@ instance (F : C ⥤ₗ Type v) : PreservesFiniteLimits (inverseAux.obj F) where
6262
noncomputable def inverse : (C ⥤ₗ Type v) ⥤ (C ⥤ₗ AddCommGrp.{v}) :=
6363
ObjectProperty.lift _ inverseAux inferInstance
6464

65+
open scoped Mon_Class
66+
6567
attribute [-instance] Functor.LaxMonoidal.comp Functor.Monoidal.instComp in
6668
/-- Implementation, see `leftExactFunctorForgetEquivalence`.
6769
This is the complicated bit, where we show that forgetting the group structure in the image of
@@ -72,10 +74,14 @@ noncomputable def unitIsoAux (F : C ⥤ AddCommGrp.{v}) [PreservesFiniteLimits F
7274
(F ⋙ forget AddCommGrp).mapCommGrp.obj (Preadditive.commGrpEquivalence.functor.obj X) := by
7375
letI : (F ⋙ forget AddCommGrp).Braided := .ofChosenFiniteProducts _
7476
letI : F.Monoidal := .ofChosenFiniteProducts _
75-
refine CommGrp_.mkIso Multiplicative.toAdd.toIso (by aesop_cat) ?_
77+
refine CommGrp_.mkIso Multiplicative.toAdd.toIso (by
78+
erw [Functor.mapCommGrp_obj_grp_one]
79+
aesop_cat) ?_
7680
dsimp [-Functor.comp_map, -ConcreteCategory.forget_map_eq_coe, -forget_map]
7781
have : F.Additive := Functor.additive_of_preserves_binary_products _
78-
rw [Functor.comp_map, F.map_add, Functor.Monoidal.μ_comp F (forget AddCommGrp) X X,
82+
simp only [Category.id_comp]
83+
erw [Functor.mapCommGrp_obj_grp_mul]
84+
erw [Functor.comp_map, F.map_add, Functor.Monoidal.μ_comp F (forget AddCommGrp) X X,
7985
Category.assoc, ← Functor.map_comp, Preadditive.comp_add, Functor.Monoidal.μ_fst,
8086
Functor.Monoidal.μ_snd]
8187
aesop_cat

Mathlib/Algebra/DualNumber.lean

Lines changed: 25 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -157,6 +157,13 @@ set_option linter.unusedVariables false in
157157
lift fe (inl a : A[ε]) = fe.val.1 a := by
158158
rw [lift_apply_apply, fst_inl, snd_inl, map_zero, zero_mul, add_zero]
159159

160+
#adaptation_note /-- https://github.com/leanprover/lean4/pull/5338
161+
The new unused variable linter flags `{fe : (A →ₐ[R] B) × B // _}`. -/
162+
set_option linter.unusedVariables false in
163+
@[simp] theorem lift_comp_inlHom (fe : {fe : (A →ₐ[R] B) × B // _}) :
164+
(lift fe).comp (inlAlgHom R A A) = fe.val.1 :=
165+
AlgHom.ext <| lift_apply_inl fe
166+
160167
#adaptation_note /-- https://github.com/leanprover/lean4/pull/5338
161168
The new unused variable linter flags `{fe : (A →ₐ[R] B) × B // _}`. -/
162169
set_option linter.unusedVariables false in
@@ -185,6 +192,24 @@ theorem lift_inlAlgHom_eps :
185192
lift ⟨(inlAlgHom _ _ _, ε), eps_mul_eps, fun _ => commute_eps_left _⟩ = AlgHom.id R A[ε] :=
186193
lift.apply_symm_apply <| AlgHom.id R A[ε]
187194

195+
@[simp]
196+
theorem range_inlAlgHom_sup_adjoin_eps :
197+
(inlAlgHom R A A).range ⊔ Algebra.adjoin R {ε} = ⊤ := by
198+
refine top_unique fun x hx => ?_; clear hx
199+
rw [← x.inl_fst_add_inr_snd_eq, inr_eq_smul_eps, ← inl_mul_eq_smul]
200+
refine add_mem ?_ (mul_mem ?_ ?_)
201+
· exact le_sup_left (α := Subalgebra R _) <| Set.mem_range_self x.fst
202+
· exact le_sup_left (α := Subalgebra R _) <| Set.mem_range_self x.snd
203+
· refine le_sup_right (α := Subalgebra R _) <| Algebra.subset_adjoin <| Set.mem_singleton ε
204+
205+
@[simp]
206+
theorem range_lift
207+
(fe : {fe : (A →ₐ[R] B) × B // fe.2 * fe.2 = 0 ∧ ∀ a, Commute fe.2 (fe.1 a)}) :
208+
(lift fe).range = fe.1.1.range ⊔ Algebra.adjoin R {fe.1.2} := by
209+
simp_rw [← Algebra.map_top, ← range_inlAlgHom_sup_adjoin_eps, Algebra.map_sup,
210+
AlgHom.map_adjoin, ← AlgHom.range_comp, Set.image_singleton, lift_apply_eps, lift_comp_inlHom,
211+
Algebra.map_top]
212+
188213
/-- Show DualNumber with values x and y as an "x + y*ε" string -/
189214
instance instRepr [Repr R] : Repr (DualNumber R) where
190215
reprPrec f p :=

Mathlib/Algebra/Group/Action/Sigma.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -28,7 +28,7 @@ namespace Sigma
2828

2929
section SMul
3030

31-
variable [∀ i, SMul M (α i)] [∀ i, SMul N (α i)] (a : M) (i : ι) (b : α i) (x : Σi, α i)
31+
variable [∀ i, SMul M (α i)] [∀ i, SMul N (α i)] (a : M) (i : ι) (b : α i) (x : Σ i, α i)
3232

3333
@[to_additive Sigma.VAdd]
3434
instance : SMul M (Σi, α i) :=

Mathlib/Algebra/Group/Ext.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -78,7 +78,7 @@ theorem RightCancelMonoid.toMonoid_injective {M : Type u} :
7878

7979
@[to_additive (attr := ext)]
8080
theorem RightCancelMonoid.ext {M : Type u} ⦃m₁ m₂ : RightCancelMonoid M⦄
81-
(h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) :
81+
(h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) :
8282
m₁ = m₂ :=
8383
RightCancelMonoid.toMonoid_injective <| Monoid.ext h_mul
8484

Mathlib/Algebra/Group/Submonoid/MulAction.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -27,7 +27,7 @@ section SetLike
2727
variable {S' : Type*} [SetLike S' M'] (s : S')
2828

2929
@[to_additive]
30-
instance (priority := low) [SMul M' α] : SMul s α where
30+
instance (priority := low) [SMul M' α] : SMul s α where
3131
smul m a := (m : M') • a
3232

3333
section MulOneClass

0 commit comments

Comments
 (0)