src/HOL/Library/Formal_Power_Series.thy
changeset 61585 a9599d3d7610
parent 61552 980dd46a03fb
child 61608 a0487caabb4a
--- a/src/HOL/Library/Formal_Power_Series.thy	Thu Nov 05 10:35:37 2015 +0100
+++ b/src/HOL/Library/Formal_Power_Series.thy	Thu Nov 05 10:39:49 2015 +0100
@@ -1323,7 +1323,7 @@
 
 subsubsection \<open>Rule 3\<close>
 
-text \<open>Rule 3 is trivial and is given by @{text fps_times_def}.\<close>
+text \<open>Rule 3 is trivial and is given by \<open>fps_times_def\<close>.\<close>
 
 
 subsubsection \<open>Rule 5 --- summation and "division" by (1 - X)\<close>
@@ -3774,7 +3774,7 @@
         unfolding eventually_nhds
         apply clarsimp
         apply (rule FalseE)
-        apply auto -- \<open>slow\<close>
+        apply auto \<comment> \<open>slow\<close>
         done
       then obtain i where "inverse (2 ^ i) < e"
         by (auto simp: eventually_sequentially)