Skip to content

Commit

Permalink
chore: classify added lemma porting notes (#10926)
Browse files Browse the repository at this point in the history
  • Loading branch information
pitmonticone committed Feb 24, 2024
1 parent 1d96f99 commit 6af752e
Show file tree
Hide file tree
Showing 3 changed files with 7 additions and 7 deletions.
10 changes: 5 additions & 5 deletions Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean
Expand Up @@ -88,11 +88,11 @@ instance : SmallCategory (WalkingMulticospan fst snd) where
assoc := by
rintro (_ | _) (_ | _) (_ | _) (_ | _) (_ | _ | _) (_ | _ | _) (_ | _ | _) <;> rfl

@[simp] -- Porting note: added simp lemma
@[simp] -- Porting note (#10756): added simp lemma
lemma Hom.id_eq_id (X : WalkingMulticospan fst snd) :
Hom.id X = 𝟙 X := rfl

@[simp] -- Porting note: added simp lemma
@[simp] -- Porting note (#10756): added simp lemma
lemma Hom.comp_eq_comp {X Y Z : WalkingMulticospan fst snd}
(f : X ⟶ Y) (g : Y ⟶ Z) : Hom.comp f g = f ≫ g := rfl

Expand Down Expand Up @@ -137,10 +137,10 @@ instance : SmallCategory (WalkingMultispan fst snd) where
assoc := by
rintro (_ | _) (_ | _) (_ | _) (_ | _) (_ | _ | _) (_ | _ | _) (_ | _ | _) <;> rfl

@[simp] -- Porting note: added simp lemma
@[simp] -- Porting note (#10756): added simp lemma
lemma Hom.id_eq_id (X : WalkingMultispan fst snd) : Hom.id X = 𝟙 X := rfl

@[simp] -- Porting note: added simp lemma
@[simp] -- Porting note (#10756): added simp lemma
lemma Hom.comp_eq_comp {X Y Z : WalkingMultispan fst snd}
(f : X ⟶ Y) (g : Y ⟶ Z) : Hom.comp f g = f ≫ g := rfl

Expand Down Expand Up @@ -549,7 +549,7 @@ theorem snd_app_right (a) : K.ι.app (WalkingMultispan.left a) = I.snd a ≫ K.
rfl
#align category_theory.limits.multicofork.snd_app_right CategoryTheory.Limits.Multicofork.snd_app_right

@[reassoc (attr := simp)] -- Porting note: added simp lemma
@[reassoc (attr := simp)] -- Porting note (#10756): added simp lemma
lemma π_comp_hom (K₁ K₂ : Multicofork I) (f : K₁ ⟶ K₂) (b : I.R) : K₁.π b ≫ f.hom = K₂.π b :=
f.w _

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Types.lean
Expand Up @@ -124,7 +124,7 @@ def sections (F : J ⥤ Type w) : Set (∀ j, F.obj j) :=
{ u | ∀ {j j'} (f : j ⟶ j'), F.map f (u j) = u j' }
#align category_theory.functor.sections CategoryTheory.Functor.sections

-- porting note: added this simp lemma
-- Porting note (#10756): added this simp lemma
@[simp]
lemma sections_property {F : J ⥤ Type w} (s : (F.sections : Type _))
{j j' : J} (f : j ⟶ j') : F.map f (s.val j) = s.val j' :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Matrix/Basic.lean
Expand Up @@ -270,7 +270,7 @@ instance distribMulAction [Monoid R] [AddMonoid α] [DistribMulAction R α] :
instance module [Semiring R] [AddCommMonoid α] [Module R α] : Module R (Matrix m n α) :=
Pi.module _ _ _

-- Porting note: added the following section with simp lemmas because `simp` fails
-- Porting note (#10756): added the following section with simp lemmas because `simp` fails
-- to apply the corresponding lemmas in the namespace `Pi`.
-- (e.g. `Pi.zero_apply` used on `OfNat.ofNat 0 i j`)
section
Expand Down

0 comments on commit 6af752e

Please sign in to comment.