Skip to content

Commit 7050e9f

Browse files
committed
chore(MvPowerSeries,PNat): avoid Coe.coe (#24945)
More along the lines of #24887
1 parent 5584925 commit 7050e9f

File tree

2 files changed

+4
-5
lines changed

2 files changed

+4
-5
lines changed

Mathlib/Data/PNat/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -211,7 +211,7 @@ def coeMonoidHom : ℕ+ →* ℕ where
211211
map_mul' := mul_coe
212212

213213
@[simp]
214-
theorem coe_coeMonoidHom : (coeMonoidHom : ℕ+ → ℕ) = Coe.coe :=
214+
theorem coe_coeMonoidHom : (coeMonoidHom : ℕ+ → ℕ) = (↑) :=
215215
rfl
216216

217217
@[simp]

Mathlib/RingTheory/MvPowerSeries/Basic.lean

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -834,11 +834,10 @@ theorem coe_X (s : σ) : ((X s : MvPolynomial σ R) : MvPowerSeries σ R) = MvPo
834834

835835
variable (σ R)
836836

837-
theorem coe_injective : Function.Injective (Coe.coe : MvPolynomial σ R → MvPowerSeries σ R) :=
838-
fun x y h => by
837+
theorem coe_injective : Function.Injective ((↑) : MvPolynomial σ R → MvPowerSeries σ R) := by
838+
intro x y h
839839
ext
840-
simp_rw [← coeff_coe]
841-
congr
840+
simp_rw [← coeff_coe, h]
842841

843842
variable {σ R φ ψ}
844843

0 commit comments

Comments
 (0)