Skip to content

Commit

Permalink
chore: classify dsimp can prove this porting notes (#10686)
Browse files Browse the repository at this point in the history
Classifies by adding issue number (#10685) to porting notes claiming `dsimp can prove this`.
  • Loading branch information
pitmonticone committed Feb 20, 2024
1 parent 89fd8bf commit 719d6e1
Show file tree
Hide file tree
Showing 7 changed files with 7 additions and 7 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Computability/TuringMachine.lean
Expand Up @@ -358,7 +358,7 @@ instance {Γ Γ'} [Inhabited Γ] [Inhabited Γ'] : Inhabited (PointedMap Γ Γ')
instance {Γ Γ'} [Inhabited Γ] [Inhabited Γ'] : CoeFun (PointedMap Γ Γ') fun _ ↦ Γ → Γ' :=
⟨PointedMap.f⟩

-- @[simp] -- Porting note: dsimp can prove this
-- @[simp] -- Porting note (#10685): dsimp can prove this
theorem PointedMap.mk_val {Γ Γ'} [Inhabited Γ] [Inhabited Γ'] (f : Γ → Γ') (pt) :
(PointedMap.mk f pt : Γ → Γ') = f :=
rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Analysis/Topology.lean
Expand Up @@ -60,7 +60,7 @@ variable (F : Ctop α σ)
instance : CoeFun (Ctop α σ) fun _ ↦ σ → Set α :=
⟨Ctop.f⟩

-- @[simp] -- Porting note: dsimp can prove this
-- @[simp] -- Porting note (#10685): dsimp can prove this
theorem coe_mk (f T h₁ I h₂ h₃ a) : (@Ctop.mk α σ f T h₁ I h₂ h₃) a = f a := rfl
#align ctop.coe_mk Ctop.coe_mk

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Multiset/Fintype.lean
Expand Up @@ -77,7 +77,7 @@ theorem Multiset.coe_eq {x y : m} : (x : α) = (y : α) ↔ x.1 = y.1 := by
rfl
#align multiset.coe_eq Multiset.coe_eq

-- @[simp] -- Porting note: dsimp can prove this
-- @[simp] -- Porting note (#10685): dsimp can prove this
theorem Multiset.coe_mk {x : α} {i : Fin (m.count x)} : ↑(m.mkToType x i) = x :=
rfl
#align multiset.coe_mk Multiset.coe_mk
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Nat/Digits.lean
Expand Up @@ -110,7 +110,7 @@ theorem digits_one (n : ℕ) : digits 1 n = List.replicate n 1 :=
rfl
#align nat.digits_one Nat.digits_one

-- @[simp] -- Porting note: dsimp can prove this
-- @[simp] -- Porting note (#10685): dsimp can prove this
theorem digits_one_succ (n : ℕ) : digits 1 (n + 1) = 1 :: digits 1 n :=
rfl
#align nat.digits_one_succ Nat.digits_one_succ
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/Subgroup/Basic.lean
Expand Up @@ -751,7 +751,7 @@ theorem coe_pow (x : H) (n : ℕ) : ((x ^ n : H) : G) = (x : G) ^ n :=
#align subgroup.coe_pow Subgroup.coe_pow
#align add_subgroup.coe_nsmul AddSubgroup.coe_nsmul

@[to_additive (attr := norm_cast)] -- Porting note: dsimp can prove this
@[to_additive (attr := norm_cast)] -- Porting note (#10685): dsimp can prove this
theorem coe_zpow (x : H) (n : ℤ) : ((x ^ n : H) : G) = (x : G) ^ n :=
rfl
#align subgroup.coe_zpow Subgroup.coe_zpow
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Function/LpSpace.lean
Expand Up @@ -186,7 +186,7 @@ theorem coeFn_mk {f : α →ₘ[μ] E} (hf : snorm f p μ < ∞) : ((⟨f, hf⟩
rfl
#align measure_theory.Lp.coe_fn_mk MeasureTheory.Lp.coeFn_mk

-- @[simp] -- Porting note: dsimp can prove this
-- @[simp] -- Porting note (#10685): dsimp can prove this
theorem coe_mk {f : α →ₘ[μ] E} (hf : snorm f p μ < ∞) : ((⟨f, hf⟩ : Lp E p μ) : α →ₘ[μ] E) = f :=
rfl
#align measure_theory.Lp.coe_mk MeasureTheory.Lp.coe_mk
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/JordanHolder.lean
Expand Up @@ -157,7 +157,7 @@ theorem step (s : CompositionSeries X) :
s.step'
#align composition_series.step CompositionSeries.step

-- @[simp] -- Porting note: dsimp can prove this
-- @[simp] -- Porting note (#10685): dsimp can prove this
theorem coeFn_mk (length : ℕ) (series step) :
(@CompositionSeries.mk X _ _ length series step : Fin length.succ → X) = series :=
rfl
Expand Down

0 comments on commit 719d6e1

Please sign in to comment.