src/HOL/Library/Polynomial.thy
changeset 61585 a9599d3d7610
parent 61260 e6f03fae14d5
child 61605 1bf7b186542e
--- a/src/HOL/Library/Polynomial.thy	Thu Nov 05 10:35:37 2015 +0100
+++ b/src/HOL/Library/Polynomial.thy	Thu Nov 05 10:39:49 2015 +0100
@@ -50,7 +50,7 @@
   "tl (x ## xs) = xs"
   by (simp add: cCons_def)
 
-subsection \<open>Definition of type @{text poly}\<close>
+subsection \<open>Definition of type \<open>poly\<close>\<close>
 
 typedef (overloaded) 'a poly = "{f :: nat \<Rightarrow> 'a::zero. \<forall>\<^sub>\<infinity> n. f n = 0}"
   morphisms coeff Abs_poly by (auto intro!: ALL_MOST)
@@ -440,7 +440,7 @@
 
 definition poly :: "'a::comm_semiring_0 poly \<Rightarrow> 'a \<Rightarrow> 'a"
 where
-  "poly p = fold_coeffs (\<lambda>a f x. a + x * f x) p (\<lambda>x. 0)" -- \<open>The Horner Schema\<close>
+  "poly p = fold_coeffs (\<lambda>a f x. a + x * f x) p (\<lambda>x. 0)" \<comment> \<open>The Horner Schema\<close>
 
 lemma poly_0 [simp]:
   "poly 0 x = 0"