Skip to content

Commit

Permalink
chore: classify dsimp cannot prove this porting notes (#10676)
Browse files Browse the repository at this point in the history
Classifies by adding issue number (#10675) to porting notes claiming `dsimp cannot prove this`.
  • Loading branch information
pitmonticone committed Feb 20, 2024
1 parent d9e8ed1 commit 90d86d7
Show file tree
Hide file tree
Showing 13 changed files with 28 additions and 28 deletions.
12 changes: 6 additions & 6 deletions Mathlib/Algebra/Free.lean
Original file line number Diff line number Diff line change
Expand Up @@ -165,7 +165,7 @@ protected def recOnPure {C : FreeMagma α → Sort l} (x) (ih1 : ∀ x, C (pure
FreeMagma.recOnMul x ih1 ih2
#align free_magma.rec_on_pure FreeMagma.recOnPure

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem map_pure (f : α → β) (x) : (f <$> pure x : FreeMagma β) = pure (f x) := rfl
#align free_magma.map_pure FreeMagma.map_pure
Expand All @@ -174,7 +174,7 @@ theorem map_pure (f : α → β) (x) : (f <$> pure x : FreeMagma β) = pure (f x
theorem map_mul' (f : α → β) (x y : FreeMagma α) : f <$> (x * y) = f <$> x * f <$> y := rfl
#align free_magma.map_mul' FreeMagma.map_mul'

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem pure_bind (f : α → FreeMagma β) (x) : pure x >>= f = f x := rfl
#align free_magma.pure_bind FreeMagma.pure_bind
Expand Down Expand Up @@ -257,7 +257,7 @@ theorem traverse_mul' :
theorem traverse_eq (x) : FreeMagma.traverse F x = traverse F x := rfl
#align free_magma.traverse_eq FreeMagma.traverse_eq

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem mul_map_seq (x y : FreeMagma α) :
((· * ·) <$> x <*> y : Id (FreeMagma α)) = (x * y : FreeMagma α) := rfl
Expand Down Expand Up @@ -588,7 +588,7 @@ def recOnPure {C : FreeSemigroup α → Sort l} (x) (ih1 : ∀ x, C (pure x))
FreeSemigroup.recOnMul x ih1 ih2
#align free_semigroup.rec_on_pure FreeSemigroup.recOnPure

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem map_pure (f : α → β) (x) : (f <$> pure x : FreeSemigroup β) = pure (f x) := rfl
#align free_semigroup.map_pure FreeSemigroup.map_pure
Expand All @@ -598,7 +598,7 @@ theorem map_mul' (f : α → β) (x y : FreeSemigroup α) : f <$> (x * y) = f <$
map_mul (map f) _ _
#align free_semigroup.map_mul' FreeSemigroup.map_mul'

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem pure_bind (f : α → FreeSemigroup β) (x) : pure x >>= f = f x := rfl
#align free_semigroup.pure_bind FreeSemigroup.pure_bind
Expand Down Expand Up @@ -674,7 +674,7 @@ end
theorem traverse_eq (x) : FreeSemigroup.traverse F x = traverse F x := rfl
#align free_semigroup.traverse_eq FreeSemigroup.traverse_eq

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem mul_map_seq (x y : FreeSemigroup α) :
((· * ·) <$> x <*> y : Id (FreeSemigroup α)) = (x * y : FreeSemigroup α) := rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Star/Free.lean
Original file line number Diff line number Diff line change
Expand Up @@ -34,7 +34,7 @@ theorem star_of (x : α) : star (of x) = of x :=
#align free_monoid.star_of FreeMonoid.star_of

/-- Note that `star_one` is already a global simp lemma, but this one works with dsimp too -/
@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
theorem star_one : star (1 : FreeMonoid α) = 1 :=
rfl
#align free_monoid.star_one FreeMonoid.star_one
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Conj.lean
Original file line number Diff line number Diff line change
Expand Up @@ -44,7 +44,7 @@ def homCongr {X Y X₁ Y₁ : C} (α : X ≅ X₁) (β : Y ≅ Y₁) : (X ⟶ Y)
rw [Category.assoc, Category.assoc, β.inv_hom_id, α.inv_hom_id_assoc, Category.comp_id]
#align category_theory.iso.hom_congr CategoryTheory.Iso.homCongr

-- @[simp, nolint simpNF] Porting note: dsimp can not prove this
-- @[simp, nolint simpNF] Porting note (#10675): dsimp can not prove this
@[simp]
theorem homCongr_apply {X Y X₁ Y₁ : C} (α : X ≅ X₁) (β : Y ≅ Y₁) (f : X ⟶ Y) :
α.homCongr β f = α.inv ≫ f ≫ β.hom := by
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean
Original file line number Diff line number Diff line change
Expand Up @@ -434,7 +434,7 @@ theorem toPiFork_π_app_zero : K.toPiFork.ι = Pi.lift K.ι :=
rfl
#align category_theory.limits.multifork.to_pi_fork_π_app_zero CategoryTheory.Limits.Multifork.toPiFork_π_app_zero

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
theorem toPiFork_π_app_one : K.toPiFork.π.app WalkingParallelPair.one = Pi.lift K.ι ≫ I.fstPiMap :=
rfl
#align category_theory.limits.multifork.to_pi_fork_π_app_one CategoryTheory.Limits.Multifork.toPiFork_π_app_one
Expand Down Expand Up @@ -464,7 +464,7 @@ theorem ofPiFork_π_app_left (c : Fork I.fstPiMap I.sndPiMap) (a) :
rfl
#align category_theory.limits.multifork.of_pi_fork_π_app_left CategoryTheory.Limits.Multifork.ofPiFork_π_app_left

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
theorem ofPiFork_π_app_right (c : Fork I.fstPiMap I.sndPiMap) (a) :
(ofPiFork I c).π.app (WalkingMulticospan.right a) = c.ι ≫ I.fstPiMap ≫ Pi.π _ _ :=
rfl
Expand Down Expand Up @@ -644,7 +644,7 @@ noncomputable def ofSigmaCofork (c : Cofork I.fstSigmaMap I.sndSigmaMap) : Multi
· simp }
#align category_theory.limits.multicofork.of_sigma_cofork CategoryTheory.Limits.Multicofork.ofSigmaCofork

-- Porting note: dsimp cannot prove this... once ofSigmaCofork_ι_app_right' is defined
-- Porting note (#10675): dsimp cannot prove this... once ofSigmaCofork_ι_app_right' is defined
@[simp, nolint simpNF]
theorem ofSigmaCofork_ι_app_left (c : Cofork I.fstSigmaMap I.sndSigmaMap) (a) :
(ofSigmaCofork I c).ι.app (WalkingMultispan.left a) =
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/Multiset/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -761,7 +761,7 @@ theorem length_toList (s : Multiset α) : s.toList.length = card s := by
rw [← coe_card, coe_toList]
#align multiset.length_to_list Multiset.length_toList

@[simp, nolint simpNF] -- Porting note: `dsimp` can not prove this, yet linter complains
@[simp, nolint simpNF] -- Porting note (#10675): `dsimp` can not prove this, yet linter complains
theorem card_zero : @card α 0 = 0 :=
rfl
#align multiset.card_zero Multiset.card_zero
Expand Down Expand Up @@ -1039,7 +1039,7 @@ theorem coe_erase (l : List α) (a : α) : erase (l : Multiset α) a = l.erase a
rfl
#align multiset.coe_erase Multiset.coe_erase

@[simp, nolint simpNF] -- Porting note: `dsimp` can not prove this, yet linter complains
@[simp, nolint simpNF] -- Porting note (#10675): `dsimp` can not prove this, yet linter complains
theorem erase_zero (a : α) : (0 : Multiset α).erase a = 0 :=
rfl
#align multiset.erase_zero Multiset.erase_zero
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/Multiset/FinsetOps.lean
Original file line number Diff line number Diff line change
Expand Up @@ -36,7 +36,7 @@ theorem coe_ndinsert (a : α) (l : List α) : ndinsert a l = (insert a l : List
rfl
#align multiset.coe_ndinsert Multiset.coe_ndinsert

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem ndinsert_zero (a : α) : ndinsert a 0 = {a} :=
rfl
#align multiset.ndinsert_zero Multiset.ndinsert_zero
Expand Down Expand Up @@ -221,7 +221,7 @@ theorem coe_ndinter (l₁ l₂ : List α) : @ndinter α _ l₁ l₂ = (l₁ ∩
rfl
#align multiset.coe_ndinter Multiset.coe_ndinter

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem zero_ndinter (s : Multiset α) : ndinter 0 s = 0 :=
rfl
#align multiset.zero_ndinter Multiset.zero_ndinter
Expand Down
12 changes: 6 additions & 6 deletions Mathlib/Data/Sum/Interval.lean
Original file line number Diff line number Diff line change
Expand Up @@ -276,7 +276,7 @@ theorem Ioc_inl_inr : Ioc (inl a₁) (inr b₂) = ∅ :=
rfl
#align sum.Ioc_inl_inr Sum.Ioc_inl_inr

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem Ioo_inl_inr : Ioo (inl a₁) (inr b₂) = ∅ := by
rfl
#align sum.Ioo_inl_inr Sum.Ioo_inl_inr
Expand All @@ -296,7 +296,7 @@ theorem Ioc_inr_inl : Ioc (inr b₁) (inl a₂) = ∅ :=
rfl
#align sum.Ioc_inr_inl Sum.Ioc_inr_inl

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem Ioo_inr_inl : Ioo (inr b₁) (inl a₂) = ∅ := by
rfl
#align sum.Ioo_inr_inl Sum.Ioo_inr_inl
Expand Down Expand Up @@ -393,19 +393,19 @@ lemma Ioc_inl_inr : Ioc (inlₗ a) (inrₗ b) = ((Ioi a).disjSum (Iic b)).map to
lemma Ioo_inl_inr : Ioo (inlₗ a) (inrₗ b) = ((Ioi a).disjSum (Iio b)).map toLex.toEmbedding := rfl
#align sum.lex.Ioo_inl_inr Sum.Lex.Ioo_inl_inr

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
lemma Icc_inr_inl : Icc (inrₗ b) (inlₗ a) = ∅ := rfl
#align sum.lex.Icc_inr_inl Sum.Lex.Icc_inr_inl

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
lemma Ico_inr_inl : Ico (inrₗ b) (inlₗ a) = ∅ := rfl
#align sum.lex.Ico_inr_inl Sum.Lex.Ico_inr_inl

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
lemma Ioc_inr_inl : Ioc (inrₗ b) (inlₗ a) = ∅ := rfl
#align sum.lex.Ioc_inr_inl Sum.Lex.Ioc_inr_inl

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
lemma Ioo_inr_inl : Ioo (inrₗ b) (inlₗ a) = ∅ := rfl
#align sum.lex.Ioo_inr_inl Sum.Lex.Ioo_inr_inl

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Vector3.lean
Original file line number Diff line number Diff line change
Expand Up @@ -266,7 +266,7 @@ theorem vectorAllP_nil (p : α → Prop) : VectorAllP p [] = True :=
rfl
#align vector_allp_nil vectorAllP_nil

@[simp, nolint simpNF] -- Porting note: dsimp cannot prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp cannot prove this
theorem vectorAllP_singleton (p : α → Prop) (x : α) : VectorAllP p (cons x []) = p x :=
rfl
#align vector_allp_singleton vectorAllP_singleton
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/FreeAbelianGroup.lean
Original file line number Diff line number Diff line change
Expand Up @@ -202,7 +202,7 @@ protected theorem induction_on' {C : FreeAbelianGroup α → Prop} (z : FreeAbel
FreeAbelianGroup.induction_on z C0 C1 Cn Cp
#align free_abelian_group.induction_on' FreeAbelianGroup.induction_on'

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem map_pure (f : α → β) (x : α) : f <$> (pure x : FreeAbelianGroup α) = pure (f x) :=
rfl
#align free_abelian_group.map_pure FreeAbelianGroup.map_pure
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/MonoidLocalization.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1757,7 +1757,7 @@ noncomputable def mulEquivOfQuotient (f : Submonoid.LocalizationMap S N) : Local

variable {f}

-- Porting note: dsimp can not prove this
-- Porting note (#10675): dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)]
theorem mulEquivOfQuotient_apply (x) : mulEquivOfQuotient f x = (monoidOf S).lift f.map_units x :=
rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/Subgroup/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -416,7 +416,7 @@ instance : SubgroupClass (Subgroup G) G where
one_mem _ := (Subgroup.toSubmonoid _).one_mem'
mul_mem := (Subgroup.toSubmonoid _).mul_mem'

@[to_additive (attr := simp, nolint simpNF)] -- Porting note: dsimp can not prove this
@[to_additive (attr := simp, nolint simpNF)] -- Porting note (#10675): dsimp can not prove this
theorem mem_carrier {s : Subgroup G} {x : G} : x ∈ s.carrier ↔ x ∈ s :=
Iff.rfl
#align subgroup.mem_carrier Subgroup.mem_carrier
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/RingTheory/Subring/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -515,7 +515,7 @@ theorem coe_intCast : ∀ n : ℤ, ((n : s) : R) = n :=
theorem coe_toSubsemiring (s : Subring R) : (s.toSubsemiring : Set R) = s :=
rfl

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem mem_toSubmonoid {s : Subring R} {x : R} : x ∈ s.toSubmonoid ↔ x ∈ s :=
Iff.rfl
#align subring.mem_to_submonoid Subring.mem_toSubmonoid
Expand All @@ -525,7 +525,7 @@ theorem coe_toSubmonoid (s : Subring R) : (s.toSubmonoid : Set R) = s :=
rfl
#align subring.coe_to_submonoid Subring.coe_toSubmonoid

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem mem_toAddSubgroup {s : Subring R} {x : R} : x ∈ s.toAddSubgroup ↔ x ∈ s :=
Iff.rfl
#align subring.mem_to_add_subgroup Subring.mem_toAddSubgroup
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/SetTheory/Ordinal/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -195,7 +195,7 @@ theorem type_def' (w : WellOrder) : ⟦w⟧ = type w.r := by
rfl
#align ordinal.type_def' Ordinal.type_def'

@[simp, nolint simpNF] -- Porting note: dsimp can not prove this
@[simp, nolint simpNF] -- Porting note (#10675): dsimp can not prove this
theorem type_def (r) [wo : IsWellOrder α r] : (⟦⟨α, r, wo⟩⟧ : Ordinal) = type r := by
rfl
#align ordinal.type_def Ordinal.type_def
Expand Down

0 comments on commit 90d86d7

Please sign in to comment.