src/HOL/SizeChange/Examples.thy
changeset 26822 67c24cfa8def
parent 25314 5eaf3e8b50a4
child 26875 e18574413bc4
--- a/src/HOL/SizeChange/Examples.thy	Wed May 07 10:59:36 2008 +0200
+++ b/src/HOL/SizeChange/Examples.thy	Wed May 07 10:59:37 2008 +0200
@@ -25,7 +25,7 @@
   apply (tactic "Sct.mk_call_graph") (* Build control graph *)
   apply (rule SCT_Main)                 (* Apply main theorem *)
   apply (simp add:finite_acg_simps) (* show finiteness *)
-  by eval (* Evaluate to true *)
+  oops (*FIXME by eval*) (* Evaluate to true *)
 
 function p :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat"
 where
@@ -42,7 +42,7 @@
   apply (tactic "Sct.mk_call_graph")
   apply (rule SCT_Main)
   apply (simp add:finite_acg_ins finite_acg_empty finite_graph_def) (* show finiteness *)
-  by eval 
+  oops (* FIXME by eval *)
 
 function foo :: "bool \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat"
 where
@@ -60,7 +60,7 @@
   apply (tactic "Sct.mk_call_graph")
   apply (rule SCT_Main)
   apply (simp add:finite_acg_ins finite_acg_empty finite_graph_def) (* show finiteness *)
-  by eval 
+  oops (* FIXME by eval *)
 
 
 function (sequential)