src/HOL/Computational_Algebra/Polynomial.thy
changeset 73114 9bf36baa8686
parent 73109 783406dd051e
child 73510 c526eb2c7ca0
equal deleted inserted replaced
73113:918f6c8b1f15 73114:9bf36baa8686
  3031 
  3031 
  3032 lemma algebraic_int_0 [simp, intro]: "algebraic_int 0"
  3032 lemma algebraic_int_0 [simp, intro]: "algebraic_int 0"
  3033   and algebraic_int_1 [simp, intro]: "algebraic_int 1"
  3033   and algebraic_int_1 [simp, intro]: "algebraic_int 1"
  3034   and algebraic_int_numeral [simp, intro]: "algebraic_int (numeral n)"
  3034   and algebraic_int_numeral [simp, intro]: "algebraic_int (numeral n)"
  3035   and algebraic_int_of_nat [simp, intro]: "algebraic_int (of_nat k)"
  3035   and algebraic_int_of_nat [simp, intro]: "algebraic_int (of_nat k)"
  3036   and algebraic_int_of_int [simp, intro]: "algebraic_int (of_int k)"
  3036   and algebraic_int_of_int [simp, intro]: "algebraic_int (of_int m)"
  3037   by (simp_all add: int_imp_algebraic_int)
  3037   by (simp_all add: int_imp_algebraic_int)
  3038 
  3038 
  3039 lemma algebraic_int_ii [simp, intro]: "algebraic_int \<i>"
  3039 lemma algebraic_int_ii [simp, intro]: "algebraic_int \<i>"
  3040 proof
  3040 proof
  3041   show "poly [:1, 0, 1:] \<i> = 0"
  3041   show "poly [:1, 0, 1:] \<i> = 0"