Skip to content

Commit 0b07d2a

Browse files
committed
chore: classify porting notes about ext (#17809)
I checked all porting notes mentioning `ext` and either fixed them (see #17810), or classified them as * #5229 if it's a new `@[ext]` lemma * #11041 if it's a regression in `ext` * #11182 if `@[ext]` had to be removed This PR should contain only modifications to comments.
1 parent a54be30 commit 0b07d2a

File tree

44 files changed

+94
-93
lines changed

Some content is hidden

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

44 files changed

+94
-93
lines changed

Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -369,7 +369,7 @@ def embeddingLiftIso (F : C ⥤ D) : embedding R C ⋙ lift R F ≅ F :=
369369
/-- Two `R`-linear functors out of the `R`-linear completion are isomorphic iff their
370370
compositions with the embedding functor are isomorphic.
371371
-/
372-
-- Porting note: used to be @[ext]
372+
-- Porting note (#11182): used to be @[ext]
373373
def ext {F G : Free R C ⥤ D} [F.Additive] [F.Linear R] [G.Additive] [G.Linear R]
374374
(α : embedding R C ⋙ F ≅ embedding R C ⋙ G) : F ≅ G :=
375375
NatIso.ofComponents (fun X => α.app X)

Mathlib/Algebra/Homology/HomologicalComplex.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -244,7 +244,7 @@ instance : Category (HomologicalComplex V c) where
244244

245245
end
246246

247-
-- Porting note: added because `Hom.ext` is not triggered automatically
247+
-- Porting note (#5229): added because `Hom.ext` is not triggered automatically
248248
@[ext]
249249
lemma hom_ext {C D : HomologicalComplex V c} (f g : C ⟶ D)
250250
(h : ∀ i, f.f i = g.f i) : f = g := by

Mathlib/Algebra/Lie/DirectSum.lean

+12-12
Original file line numberDiff line numberDiff line change
@@ -43,13 +43,13 @@ variable [∀ i, LieRingModule L (M i)] [∀ i, LieModule R L (M i)]
4343
instance : LieRingModule L (⨁ i, M i) where
4444
bracket x m := m.mapRange (fun _ m' => ⁅x, m'⁆) fun _ => lie_zero x
4545
add_lie x y m := by
46-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
46+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
4747
simp only [mapRange_apply, add_apply, add_lie]
4848
lie_add x m n := by
49-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
49+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
5050
simp only [mapRange_apply, add_apply, lie_add]
5151
leibniz_lie x y m := by
52-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
52+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
5353
simp only [mapRange_apply, lie_lie, add_apply, sub_add_cancel]
5454

5555
@[simp]
@@ -58,10 +58,10 @@ theorem lie_module_bracket_apply (x : L) (m : ⨁ i, M i) (i : ι) : ⁅x, m⁆
5858

5959
instance : LieModule R L (⨁ i, M i) where
6060
smul_lie t x m := by
61-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext i`
61+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext i`
6262
simp only [smul_lie, lie_module_bracket_apply, smul_apply]
6363
lie_smul t x m := by
64-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext i`
64+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext i`
6565
simp only [lie_smul, lie_module_bracket_apply, smul_apply]
6666

6767
variable (R ι L M)
@@ -70,7 +70,7 @@ variable (R ι L M)
7070
def lieModuleOf [DecidableEq ι] (j : ι) : M j →ₗ⁅R,L⁆ ⨁ i, M i :=
7171
{ lof R ι M j with
7272
map_lie' := fun {x m} => by
73-
refine DFinsupp.ext fun i => ?_ -- Porting note: Originally `ext i`
73+
refine DFinsupp.ext fun i => ?_ -- Porting note (#11041): Originally `ext i`
7474
by_cases h : j = i
7575
· rw [← h]; simp
7676
· -- This used to be the end of the proof before leanprover/lean4#2644
@@ -98,16 +98,16 @@ instance lieRing : LieRing (⨁ i, L i) :=
9898
{ (inferInstance : AddCommGroup _) with
9999
bracket := zipWith (fun _ => fun x y => ⁅x, y⁆) fun _ => lie_zero 0
100100
add_lie := fun x y z => by
101-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
101+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
102102
simp only [zipWith_apply, add_apply, add_lie]
103103
lie_add := fun x y z => by
104-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
104+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
105105
simp only [zipWith_apply, add_apply, lie_add]
106106
lie_self := fun x => by
107-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
107+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
108108
simp only [zipWith_apply, add_apply, lie_self, zero_apply]
109109
leibniz_lie := fun x y z => by
110-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
110+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
111111
simp only [sub_apply, zipWith_apply, add_apply, zero_apply]
112112
apply leibniz_lie }
113113

@@ -137,7 +137,7 @@ theorem lie_of [DecidableEq ι] {i j : ι} (x : L i) (y : L j) :
137137
instance lieAlgebra : LieAlgebra R (⨁ i, L i) :=
138138
{ (inferInstance : Module R _) with
139139
lie_smul := fun c x y => by
140-
refine DFinsupp.ext fun _ => ?_ -- Porting note: Originally `ext`
140+
refine DFinsupp.ext fun _ => ?_ -- Porting note (#11041): Originally `ext`
141141
simp only [zipWith_apply, smul_apply, bracket_apply, lie_smul] }
142142

143143
variable (R ι)
@@ -148,7 +148,7 @@ def lieAlgebraOf [DecidableEq ι] (j : ι) : L j →ₗ⁅R⁆ ⨁ i, L i :=
148148
{ lof R ι L j with
149149
toFun := of L j
150150
map_lie' := fun {x y} => by
151-
refine DFinsupp.ext fun i => ?_ -- Porting note: Originally `ext i`
151+
refine DFinsupp.ext fun i => ?_ -- Porting note (#11041): Originally `ext i`
152152
by_cases h : j = i
153153
· rw [← h]
154154
-- This used to be the end of the proof before leanprover/lean4#2644

Mathlib/Algebra/MonoidAlgebra/Basic.lean

+5-5
Original file line numberDiff line numberDiff line change
@@ -90,7 +90,7 @@ def liftMagma [Module k A] [IsScalarTower k A A] [SMulCommClass k A A] :
9090
sum_single_index, Function.comp_apply, one_smul, zero_smul, MulHom.coe_comp,
9191
NonUnitalAlgHom.coe_to_mulHom]
9292
right_inv F := by
93-
-- Porting note: `ext` → `refine nonUnitalAlgHom_ext' k (MulHom.ext fun m => ?_)`
93+
-- Porting note (#11041): `ext` → `refine nonUnitalAlgHom_ext' k (MulHom.ext fun m => ?_)`
9494
refine nonUnitalAlgHom_ext' k (MulHom.ext fun m => ?_)
9595
simp only [NonUnitalAlgHom.coe_mk, ofMagma_apply, NonUnitalAlgHom.toMulHom_eq_coe,
9696
sum_single_index, Function.comp_apply, one_smul, zero_smul, MulHom.coe_comp,
@@ -109,7 +109,7 @@ In particular this provides the instance `Algebra k (MonoidAlgebra k G)`.
109109
instance algebra {A : Type*} [CommSemiring k] [Semiring A] [Algebra k A] [Monoid G] :
110110
Algebra k (MonoidAlgebra A G) :=
111111
{ singleOneRingHom.comp (algebraMap k A) with
112-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
112+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
113113
smul_def' := fun r a => by
114114
refine Finsupp.ext fun _ => ?_
115115
-- Porting note: Newly required.
@@ -125,7 +125,7 @@ def singleOneAlgHom {A : Type*} [CommSemiring k] [Semiring A] [Algebra k A] [Mon
125125
A →ₐ[k] MonoidAlgebra A G :=
126126
{ singleOneRingHom with
127127
commutes' := fun r => by
128-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
128+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
129129
refine Finsupp.ext fun _ => ?_
130130
simp
131131
rfl }
@@ -390,7 +390,7 @@ In particular this provides the instance `Algebra k k[G]`.
390390
instance algebra [CommSemiring R] [Semiring k] [Algebra R k] [AddMonoid G] :
391391
Algebra R k[G] :=
392392
{ singleZeroRingHom.comp (algebraMap R k) with
393-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
393+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
394394
smul_def' := fun r a => by
395395
refine Finsupp.ext fun _ => ?_
396396
-- Porting note: Newly required.
@@ -405,7 +405,7 @@ instance algebra [CommSemiring R] [Semiring k] [Algebra R k] [AddMonoid G] :
405405
def singleZeroAlgHom [CommSemiring R] [Semiring k] [Algebra R k] [AddMonoid G] : k →ₐ[R] k[G] :=
406406
{ singleZeroRingHom with
407407
commutes' := fun r => by
408-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
408+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
409409
refine Finsupp.ext fun _ => ?_
410410
simp
411411
rfl }

Mathlib/Algebra/MonoidAlgebra/Defs.lean

+6-6
Original file line numberDiff line numberDiff line change
@@ -563,7 +563,7 @@ theorem liftNC_smul [MulOneClass G] {R : Type*} [Semiring R] (f : k →+* R) (g
563563
suffices (liftNC (↑f) g).comp (smulAddHom k (MonoidAlgebra k G) c) =
564564
(AddMonoidHom.mulLeft (f c)).comp (liftNC (↑f) g) from
565565
DFunLike.congr_fun this φ
566-
-- Porting note: `ext` couldn't a find appropriate theorem.
566+
-- Porting note (#11041): `ext` couldn't a find appropriate theorem.
567567
refine addHom_ext' fun a => AddMonoidHom.ext fun b => ?_
568568
-- Porting note: `reducible` cannot be `local` so the proof gets more complex.
569569
unfold MonoidAlgebra
@@ -584,7 +584,7 @@ variable (k) [Semiring k] [DistribSMul R k] [Mul G]
584584
instance isScalarTower_self [IsScalarTower R k k] :
585585
IsScalarTower R (MonoidAlgebra k G) (MonoidAlgebra k G) :=
586586
fun t a b => by
587-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
587+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
588588
refine Finsupp.ext fun m => ?_
589589
-- Porting note: `refine` & `rw` are required because `simp` behaves differently.
590590
classical
@@ -600,7 +600,7 @@ also commute with the algebra multiplication. -/
600600
instance smulCommClass_self [SMulCommClass R k k] :
601601
SMulCommClass R (MonoidAlgebra k G) (MonoidAlgebra k G) :=
602602
fun t a b => by
603-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
603+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
604604
refine Finsupp.ext fun m => ?_
605605
-- Porting note: `refine` & `rw` are required because `simp` behaves differently.
606606
classical
@@ -742,7 +742,7 @@ protected noncomputable def opRingEquiv [Monoid G] :
742742
rw [← AddEquiv.coe_toAddMonoidHom]
743743
refine Iff.mpr (AddMonoidHom.map_mul_iff (R := (MonoidAlgebra k G)ᵐᵒᵖ)
744744
(S := MonoidAlgebra kᵐᵒᵖ Gᵐᵒᵖ) _) ?_
745-
-- Porting note: Was `ext`.
745+
-- Porting note (#11041): Was `ext`.
746746
refine AddMonoidHom.mul_op_ext _ _ <| addHom_ext' fun i₁ => AddMonoidHom.ext fun r₁ =>
747747
AddMonoidHom.mul_op_ext _ _ <| addHom_ext' fun i₂ => AddMonoidHom.ext fun r₂ => ?_
748748
-- Porting note: `reducible` cannot be `local` so proof gets long.
@@ -924,7 +924,7 @@ instance nonUnitalNonAssocSemiring : NonUnitalNonAssocSemiring k[G] :=
924924
simp only [mul_def]
925925
exact Eq.trans (congr_arg (sum f) (funext₂ fun a₁ b₁ => sum_zero_index)) sum_zero
926926
nsmul := fun n f => n • f
927-
-- Porting note: `ext` → `refine Finsupp.ext fun _ => ?_`
927+
-- Porting note (#11041): `ext` → `refine Finsupp.ext fun _ => ?_`
928928
nsmul_zero := by
929929
intros
930930
refine Finsupp.ext fun _ => ?_
@@ -1399,7 +1399,7 @@ protected noncomputable def opRingEquiv [AddCommMonoid G] :
13991399
rw [Equiv.toFun_as_coe, AddEquiv.toEquiv_eq_coe]; erw [AddEquiv.coe_toEquiv]
14001400
rw [← AddEquiv.coe_toAddMonoidHom]
14011401
refine Iff.mpr (AddMonoidHom.map_mul_iff (R := k[G]ᵐᵒᵖ) (S := kᵐᵒᵖ[G]) _) ?_
1402-
-- Porting note: Was `ext`.
1402+
-- Porting note (#11041): Was `ext`.
14031403
refine AddMonoidHom.mul_op_ext _ _ <| addHom_ext' fun i₁ => AddMonoidHom.ext fun r₁ =>
14041404
AddMonoidHom.mul_op_ext _ _ <| addHom_ext' fun i₂ => AddMonoidHom.ext fun r₂ => ?_
14051405
-- Porting note: `reducible` cannot be `local` so proof gets long.

Mathlib/Algebra/MonoidAlgebra/Division.lean

+7-7
Original file line numberDiff line numberDiff line change
@@ -69,14 +69,14 @@ theorem zero_divOf (g : G) : (0 : k[G]) /ᵒᶠ g = 0 :=
6969

7070
@[simp]
7171
theorem divOf_zero (x : k[G]) : x /ᵒᶠ 0 = x := by
72-
refine Finsupp.ext fun _ => ?_ -- Porting note: `ext` doesn't work
72+
refine Finsupp.ext fun _ => ?_ -- Porting note (#11041): `ext` doesn't work
7373
simp only [AddMonoidAlgebra.divOf_apply, zero_add]
7474

7575
theorem add_divOf (x y : k[G]) (g : G) : (x + y) /ᵒᶠ g = x /ᵒᶠ g + y /ᵒᶠ g :=
7676
map_add (Finsupp.comapDomain.addMonoidHom _) _ _
7777

7878
theorem divOf_add (x : k[G]) (a b : G) : x /ᵒᶠ (a + b) = x /ᵒᶠ a /ᵒᶠ b := by
79-
refine Finsupp.ext fun _ => ?_ -- Porting note: `ext` doesn't work
79+
refine Finsupp.ext fun _ => ?_ -- Porting note (#11041): `ext` doesn't work
8080
simp only [AddMonoidAlgebra.divOf_apply, add_assoc]
8181

8282
/-- A bundled version of `AddMonoidAlgebra.divOf`. -/
@@ -93,13 +93,13 @@ noncomputable def divOfHom : Multiplicative G →* AddMonoid.End k[G] where
9393
(divOf_add _ _ _)
9494

9595
theorem of'_mul_divOf (a : G) (x : k[G]) : of' k G a * x /ᵒᶠ a = x := by
96-
refine Finsupp.ext fun _ => ?_ -- Porting note: `ext` doesn't work
96+
refine Finsupp.ext fun _ => ?_ -- Porting note (#11041): `ext` doesn't work
9797
rw [AddMonoidAlgebra.divOf_apply, of'_apply, single_mul_apply_aux, one_mul]
9898
intro c
9999
exact add_right_inj _
100100

101101
theorem mul_of'_divOf (x : k[G]) (a : G) : x * of' k G a /ᵒᶠ a = x := by
102-
refine Finsupp.ext fun _ => ?_ -- Porting note: `ext` doesn't work
102+
refine Finsupp.ext fun _ => ?_ -- Porting note (#11041): `ext` doesn't work
103103
rw [AddMonoidAlgebra.divOf_apply, of'_apply, mul_single_apply_aux, mul_one]
104104
intro c
105105
rw [add_comm]
@@ -134,14 +134,14 @@ theorem modOf_apply_self_add (x : k[G]) (g : G) (d : G) : (x %ᵒᶠ g) (g + d)
134134
modOf_apply_of_exists_add _ _ _ ⟨_, rfl⟩
135135

136136
theorem of'_mul_modOf (g : G) (x : k[G]) : of' k G g * x %ᵒᶠ g = 0 := by
137-
refine Finsupp.ext fun g' => ?_ -- Porting note: `ext g'` doesn't work
137+
refine Finsupp.ext fun g' => ?_ -- Porting note (#11041): `ext g'` doesn't work
138138
rw [Finsupp.zero_apply]
139139
obtain ⟨d, rfl⟩ | h := em (∃ d, g' = g + d)
140140
· rw [modOf_apply_self_add]
141141
· rw [modOf_apply_of_not_exists_add _ _ _ h, of'_apply, single_mul_apply_of_not_exists_add _ _ h]
142142

143143
theorem mul_of'_modOf (x : k[G]) (g : G) : x * of' k G g %ᵒᶠ g = 0 := by
144-
refine Finsupp.ext fun g' => ?_ -- Porting note: `ext g'` doesn't work
144+
refine Finsupp.ext fun g' => ?_ -- Porting note (#11041): `ext g'` doesn't work
145145
rw [Finsupp.zero_apply]
146146
obtain ⟨d, rfl⟩ | h := em (∃ d, g' = g + d)
147147
· rw [modOf_apply_self_add]
@@ -153,7 +153,7 @@ theorem of'_modOf (g : G) : of' k G g %ᵒᶠ g = 0 := by
153153

154154
theorem divOf_add_modOf (x : k[G]) (g : G) :
155155
of' k G g * (x /ᵒᶠ g) + x %ᵒᶠ g = x := by
156-
refine Finsupp.ext fun g' => ?_ -- Porting note: `ext` doesn't work
156+
refine Finsupp.ext fun g' => ?_ -- Porting note (#11041): `ext` doesn't work
157157
rw [Finsupp.add_apply] -- Porting note: changed from `simp_rw` which can't see through the type
158158
obtain ⟨d, rfl⟩ | h := em (∃ d, g' = g + d)
159159
swap

Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -129,7 +129,7 @@ theorem toDirectSum_mul [DecidableEq ι] [AddMonoid ι] [Semiring M] (f g : AddM
129129
let _ : NonUnitalNonAssocSemiring (ι →₀ M) := AddMonoidAlgebra.nonUnitalNonAssocSemiring
130130
revert f g
131131
rw [AddMonoidHom.map_mul_iff]
132-
-- Porting note: does not find `addHom_ext'`, was `ext (xi xv yi yv) : 4`
132+
-- Porting note (#11041): does not find `addHom_ext'`, was `ext (xi xv yi yv) : 4`
133133
refine Finsupp.addHom_ext' fun xi => AddMonoidHom.ext fun xv => ?_
134134
refine Finsupp.addHom_ext' fun yi => AddMonoidHom.ext fun yv => ?_
135135
dsimp only [AddMonoidHom.comp_apply, AddMonoidHom.compl₂_apply, AddMonoidHom.compr₂_apply,

Mathlib/Algebra/MvPolynomial/Basic.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -404,12 +404,12 @@ theorem induction_on {M : MvPolynomial σ R → Prop} (p : MvPolynomial σ R) (h
404404
theorem ringHom_ext {A : Type*} [Semiring A] {f g : MvPolynomial σ R →+* A}
405405
(hC : ∀ r, f (C r) = g (C r)) (hX : ∀ i, f (X i) = g (X i)) : f = g := by
406406
refine AddMonoidAlgebra.ringHom_ext' ?_ ?_
407-
-- Porting note: this has high priority, but Lean still chooses `RingHom.ext`, why?
407+
-- Porting note (#11041): this has high priority, but Lean still chooses `RingHom.ext`, why?
408408
-- probably because of the type synonym
409409
· ext x
410410
exact hC _
411411
· apply Finsupp.mulHom_ext'; intros x
412-
-- Porting note: `Finsupp.mulHom_ext'` needs to have increased priority
412+
-- Porting note (#11041): `Finsupp.mulHom_ext'` needs to have increased priority
413413
apply MonoidHom.ext_mnat
414414
exact hX _
415415

Mathlib/Algebra/Polynomial/Laurent.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -87,7 +87,7 @@ scoped[LaurentPolynomial] notation:9000 R "[T;T⁻¹]" => LaurentPolynomial R
8787

8888
open LaurentPolynomial
8989

90-
-- Porting note: `ext` no longer applies `Finsupp.ext` automatically
90+
-- Porting note (#5229): `ext` no longer applies `Finsupp.ext` automatically
9191
@[ext]
9292
theorem LaurentPolynomial.ext [Semiring R] {p q : R[T;T⁻¹]} (h : ∀ a, p a = q a) : p = q :=
9393
Finsupp.ext h

Mathlib/AlgebraicGeometry/Restrict.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -392,13 +392,13 @@ theorem image_morphismRestrict_preimage {X Y : Scheme.{u}} (f : X ⟶ Y) (U : Y.
392392
-- Porting note: this rewrite was not necessary
393393
rw [SetLike.mem_coe]
394394
convert hx'
395-
-- Porting note: `ext1` is not compiling
395+
-- Porting note (#11041): `ext1` is not compiling
396396
refine Subtype.ext ?_
397397
exact (morphismRestrict_base_coe f U ⟨x, hx⟩).symm
398398
· rintro ⟨⟨x, hx⟩, hx' : _ ∈ V.1, rfl : x = _⟩
399399
refine ⟨⟨_, hx⟩, (?_ : (f ∣_ U).base ⟨x, hx⟩ ∈ V.1), rfl⟩
400400
convert hx'
401-
-- Porting note: `ext1` is compiling
401+
-- Porting note (#11041): `ext1` is compiling
402402
refine Subtype.ext ?_
403403
exact morphismRestrict_base_coe f U ⟨x, hx⟩
404404

Mathlib/AlgebraicGeometry/Spec.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -287,7 +287,7 @@ instance isIso_toSpecΓ (R : CommRingCat.{u}) : IsIso (toSpecΓ R) := by
287287
@[reassoc]
288288
theorem Spec_Γ_naturality {R S : CommRingCat.{u}} (f : R ⟶ S) :
289289
f ≫ toSpecΓ S = toSpecΓ R ≫ Γ.map (Spec.toLocallyRingedSpace.map f.op).op := by
290-
-- Porting note: `ext` failed to pick up one of the three lemmas
290+
-- Porting note (#11041): `ext` failed to pick up one of the three lemmas
291291
refine RingHom.ext fun x => Subtype.ext <| funext fun x' => ?_; symm
292292
apply Localization.localRingHom_to_map
293293

Mathlib/AlgebraicTopology/SimplexCategory.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -142,7 +142,7 @@ lemma id_toOrderHom (a : SimplexCategory) :
142142
lemma comp_toOrderHom {a b c : SimplexCategory} (f : a ⟶ b) (g : b ⟶ c) :
143143
(f ≫ g).toOrderHom = g.toOrderHom.comp f.toOrderHom := rfl
144144

145-
-- Porting note: added because `Hom.ext'` is not triggered automatically
145+
-- Porting note (#5229): added because `Hom.ext'` is not triggered automatically
146146
@[ext]
147147
theorem Hom.ext {a b : SimplexCategory} (f g : a ⟶ b) :
148148
f.toOrderHom = g.toOrderHom → f = g :=

Mathlib/AlgebraicTopology/SplitSimplicialObject.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -351,7 +351,7 @@ variable {C}
351351

352352
namespace Split
353353

354-
-- Porting note: added as `Hom.ext` is not triggered automatically
354+
-- Porting note (#5229): added as `Hom.ext` is not triggered automatically
355355
@[ext]
356356
theorem hom_ext {S₁ S₂ : Split C} (Φ₁ Φ₂ : S₁ ⟶ S₂) (h : ∀ n : ℕ, Φ₁.f n = Φ₂.f n) : Φ₁ = Φ₂ :=
357357
Hom.ext _ _ h

Mathlib/CategoryTheory/Abelian/Pseudoelements.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -258,7 +258,7 @@ theorem zero_morphism_ext {P Q : C} (f : P ⟶ Q) : (∀ a, f a = 0) → f = 0 :
258258
theorem zero_morphism_ext' {P Q : C} (f : P ⟶ Q) : (∀ a, f a = 0) → 0 = f :=
259259
Eq.symm ∘ zero_morphism_ext f
260260

261-
-- Porting note: these are no longer valid as `ext` lemmas.
261+
-- Porting note (#11182): these are no longer valid as `ext` lemmas.
262262
-- scoped[Pseudoelement]
263263
-- attribute [ext]
264264
-- CategoryTheory.Abelian.Pseudoelement.zero_morphism_ext

Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -245,7 +245,7 @@ instance category (F G : OplaxFunctor B C) : Category (F ⟶ G) where
245245
id := Modification.id
246246
comp := Modification.vcomp
247247

248-
-- Porting note: duplicating the `ext` lemma.
248+
-- Porting note (#5229): duplicating the `ext` lemma.
249249
@[ext]
250250
lemma ext {F G : OplaxFunctor B C} {α β : F ⟶ G} {m n : α ⟶ β} (w : ∀ b, m.app b = n.app b) :
251251
m = n := by

Mathlib/CategoryTheory/Closed/Functor.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -79,14 +79,14 @@ theorem expComparison_ev (A B : C) :
7979
Limits.prod.map (𝟙 (F.obj A)) ((expComparison F A).app B) ≫ (exp.ev (F.obj A)).app (F.obj B) =
8080
inv (prodComparison F _ _) ≫ F.map ((exp.ev _).app _) := by
8181
convert mateEquiv_counit _ _ (prodComparisonNatIso F A).inv B using 2
82-
apply IsIso.inv_eq_of_hom_inv_id -- Porting note: was `ext`
82+
apply IsIso.inv_eq_of_hom_inv_id -- Porting note (#11041): was `ext`
8383
simp only [Limits.prodComparisonNatIso_inv, asIso_inv, NatIso.isIso_inv_app, IsIso.hom_inv_id]
8484

8585
theorem coev_expComparison (A B : C) :
8686
F.map ((exp.coev A).app B) ≫ (expComparison F A).app (A ⨯ B) =
8787
(exp.coev _).app (F.obj B) ≫ (exp (F.obj A)).map (inv (prodComparison F A B)) := by
8888
convert unit_mateEquiv _ _ (prodComparisonNatIso F A).inv B using 3
89-
apply IsIso.inv_eq_of_hom_inv_id -- Porting note: was `ext`
89+
apply IsIso.inv_eq_of_hom_inv_id -- Porting note (#11041): was `ext`
9090
dsimp
9191
simp
9292

Mathlib/CategoryTheory/Comma/Basic.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -106,7 +106,7 @@ section
106106

107107
variable {X Y Z : Comma L R} {f : X ⟶ Y} {g : Y ⟶ Z}
108108

109-
-- Porting note: this lemma was added because `CommaMorphism.ext`
109+
-- Porting note (#5229): this lemma was added because `CommaMorphism.ext`
110110
-- was not triggered automatically
111111
@[ext]
112112
lemma hom_ext (f g : X ⟶ Y) (h₁ : f.left = g.left) (h₂ : f.right = g.right) : f = g :=

0 commit comments

Comments
 (0)