doc-src/Codegen/Thy/Inductive_Predicate.thy
changeset 39065 16a2ed09217a
parent 38811 c3511b112595
child 39682 066e2d4d0de8
--- a/doc-src/Codegen/Thy/Inductive_Predicate.thy	Thu Sep 02 16:41:42 2010 +0200
+++ b/doc-src/Codegen/Thy/Inductive_Predicate.thy	Thu Sep 02 16:41:42 2010 +0200
@@ -220,8 +220,8 @@
   "values"} and the number of elements.
 *}
 
-values %quote [mode: i \<Rightarrow> o \<Rightarrow> bool] 20 "{n. tranclp succ 10 n}"
-values %quote [mode: o \<Rightarrow> i \<Rightarrow> bool] 10 "{n. tranclp succ n 10}"
+values %quote [mode: i \<Rightarrow> o \<Rightarrow> bool] 1 "{n. tranclp succ 10 n}" (*FIMXE does not terminate for n\<ge>1*)
+values %quote [mode: o \<Rightarrow> i \<Rightarrow> bool] 1 "{n. tranclp succ n 10}"
 
 
 subsection {* Embedding into functional code within Isabelle/HOL *}