Zulip Chat Archive
Stream: new members
Topic: simple polynomial
vxctyxeha (Apr 16 2025 at 08:30):
how to solve this problem
import Mathlib
open Polynomial
attribute [local simp] coeff_X
lemma coeff : Polynomial.coeff (1 : ℤ[X]) 2 = 0 := by
Ruben Van de Velde (Apr 16 2025 at 08:34):
What have you tried?
Bolton Bailey (Apr 16 2025 at 21:48):
This works:
import Mathlib
open Polynomial
attribute [local simp] coeff_X
lemma coeff : Polynomial.coeff (1 : ℤ[X]) 2 = 0 := by
have : (1 : ℤ[X]) = Polynomial.C 1 := by exact rfl
rw [this, Polynomial.coeff_C]
simp
Last updated: May 02 2025 at 03:31 UTC