File tree 2 files changed +2
-2
lines changed
RingTheory/FractionalIdeal
2 files changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -249,7 +249,7 @@ def Functor.mapHomotopyCategory (F : V ⥤ W) [F.Additive] (c : ComplexShape ι)
249
249
(fun _ _ _ _ ⟨h⟩ => HomotopyCategory.eq_of_homotopy _ _ (F.mapHomotopy h))
250
250
#align category_theory.functor.map_homotopy_category CategoryTheory.Functor.mapHomotopyCategory
251
251
252
- -- porting note: added this lemma because of the new definition of `Functor.mapHomotopyCategory`
252
+ -- Porting note (#10756) : added lemma because of new definition of `Functor.mapHomotopyCategory`
253
253
@[simp]
254
254
lemma Functor.mapHomotopyCategory_map (F : V ⥤ W) [F.Additive] {c : ComplexShape ι}
255
255
{K L : HomologicalComplex V c} (f : K ⟶ L) :
Original file line number Diff line number Diff line change @@ -208,7 +208,7 @@ theorem coe_mk (I : Submodule R P) (hI : IsFractional S I) :
208
208
rfl
209
209
#align fractional_ideal.coe_mk FractionalIdeal.coe_mk
210
210
211
- -- Porting note: added this lemma because Lean can't see through the composition of coercions.
211
+ -- Porting note (#10756) : added lemma because Lean can't see through the composition of coercions.
212
212
theorem coeToSet_coeToSubmodule (I : FractionalIdeal S P) :
213
213
((I : Submodule R P) : Set P) = I :=
214
214
rfl
You can’t perform that action at this time.
0 commit comments