src/HOL/Decision_Procs/ex/Approximation_Quickcheck_Ex.thy
changeset 69597 ff784d5a5bfb
parent 67443 3abf6a722518
--- a/src/HOL/Decision_Procs/ex/Approximation_Quickcheck_Ex.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Decision_Procs/ex/Approximation_Quickcheck_Ex.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -31,7 +31,7 @@
   shows "x > 1 \<Longrightarrow> x \<le> 2 ^ 20 * log 2 x + 1 \<and> (sin x)\<^sup>2 + (cos x)\<^sup>2 = 1"
   using [[quickcheck_approximation_custom_seed = 1]]
   using [[quickcheck_approximation_epsilon = 0.00000001]]
-    \<comment> \<open>avoids spurious counterexamples in approximate computation of @{term "(sin x)\<^sup>2 + (cos x)\<^sup>2"}
+    \<comment> \<open>avoids spurious counterexamples in approximate computation of \<^term>\<open>(sin x)\<^sup>2 + (cos x)\<^sup>2\<close>
       and therefore avoids expensive failing attempts for certification\<close>
   quickcheck[approximation, expect=counterexample, size=20]
   oops