src/HOL/Library/Polynomial.thy
changeset 63145 703edebd1d92
parent 63060 293ede07b775
child 63317 ca187a9f66da
equal deleted inserted replaced
63143:ef72b104fa32 63145:703edebd1d92
   441 lemma is_zero_null [code_abbrev]:
   441 lemma is_zero_null [code_abbrev]:
   442   "is_zero p \<longleftrightarrow> p = 0"
   442   "is_zero p \<longleftrightarrow> p = 0"
   443   by (simp add: is_zero_def null_def)
   443   by (simp add: is_zero_def null_def)
   444 
   444 
   445 subsubsection \<open>Reconstructing the polynomial from the list\<close>
   445 subsubsection \<open>Reconstructing the polynomial from the list\<close>
   446   -- \<open>contributed by Sebastiaan J.C. Joosten and René Thiemann\<close>
   446   \<comment> \<open>contributed by Sebastiaan J.C. Joosten and René Thiemann\<close>
   447 
   447 
   448 definition poly_of_list :: "'a::comm_monoid_add list \<Rightarrow> 'a poly"
   448 definition poly_of_list :: "'a::comm_monoid_add list \<Rightarrow> 'a poly"
   449 where
   449 where
   450   [simp]: "poly_of_list = Poly"
   450   [simp]: "poly_of_list = Poly"
   451 
   451