Commit 2023-03-08 07:29 301a5b54

View on Github →

feat: port Data.Polynomial.Basic (#2620)

Estimated changes

added def Polynomial.C
added theorem Polynomial.C_0
added theorem Polynomial.C_1
added theorem Polynomial.C_add
added theorem Polynomial.C_bit0
added theorem Polynomial.C_bit1
added theorem Polynomial.C_eq_zero
added theorem Polynomial.C_inj
added theorem Polynomial.C_injective
added theorem Polynomial.C_mul
added theorem Polynomial.C_ne_zero
added theorem Polynomial.C_pow
added def Polynomial.X
added theorem Polynomial.X_mul
added theorem Polynomial.X_mul_C
added theorem Polynomial.X_ne_zero
added theorem Polynomial.X_pow_mul
added theorem Polynomial.X_pow_mul_C
added theorem Polynomial.addHom_ext'
added theorem Polynomial.addHom_ext
added def Polynomial.coeff
added theorem Polynomial.coeff_C
added theorem Polynomial.coeff_X
added theorem Polynomial.coeff_X_one
added theorem Polynomial.coeff_erase
added theorem Polynomial.coeff_inj
added theorem Polynomial.coeff_neg
added theorem Polynomial.coeff_sub
added theorem Polynomial.coeff_zero
added theorem Polynomial.commute_X
added theorem Polynomial.erase_ne
added theorem Polynomial.erase_same
added theorem Polynomial.erase_zero
added theorem Polynomial.eta
added theorem Polynomial.ext
added theorem Polynomial.ext_iff
added theorem Polynomial.lhom_ext'
added theorem Polynomial.smul_C
added def Polynomial.sum
added theorem Polynomial.sum_C_index
added theorem Polynomial.sum_X_index
added theorem Polynomial.sum_add'
added theorem Polynomial.sum_add
added theorem Polynomial.sum_def
added theorem Polynomial.support_X
added theorem Polynomial.support_add
added theorem Polynomial.support_neg
added theorem Polynomial.toFinsupp_C
added theorem Polynomial.toFinsupp_X
added structure Polynomial