File tree Expand file tree Collapse file tree 2 files changed +4
-5
lines changed Expand file tree Collapse file tree 2 files changed +4
-5
lines changed Original file line number Diff line number Diff line change @@ -211,7 +211,7 @@ def coeMonoidHom : ℕ+ →* ℕ where
211
211
map_mul' := mul_coe
212
212
213
213
@[simp]
214
- theorem coe_coeMonoidHom : (coeMonoidHom : ℕ+ → ℕ) = Coe.coe :=
214
+ theorem coe_coeMonoidHom : (coeMonoidHom : ℕ+ → ℕ) = (↑) :=
215
215
rfl
216
216
217
217
@[simp]
Original file line number Diff line number Diff line change @@ -834,11 +834,10 @@ theorem coe_X (s : σ) : ((X s : MvPolynomial σ R) : MvPowerSeries σ R) = MvPo
834
834
835
835
variable (σ R)
836
836
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
839
839
ext
840
- simp_rw [← coeff_coe]
841
- congr
840
+ simp_rw [← coeff_coe, h]
842
841
843
842
variable {σ R φ ψ}
844
843
You can’t perform that action at this time.
0 commit comments