src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy
changeset 39195 5ab54bf226ac
parent 38664 7215ae18f44b
child 39254 344d97e7b342
--- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy	Tue Sep 07 11:51:53 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy	Tue Sep 07 11:51:53 2010 +0200
@@ -810,8 +810,7 @@
  (let (y', x') = f i y x; (y'', xs') = fold_map_idx f (Suc i) y' xs
  in (y'', x' # xs'))"
 
-text {* mode analysis explores thousand modes - this is infeasible at the moment... *}
-(*code_pred [inductify, show_steps] fold_map_idx .*)
+code_pred [inductify] fold_map_idx .
 
 subsection {* Minimum *}
 
@@ -939,10 +938,10 @@
 "height ET = 0"
 | "height (MKT x l r h) = max (height l) (height r) + 1"
 
-consts avl :: "'a tree => bool"
-primrec
+primrec avl :: "'a tree => bool"
+where
   "avl ET = True"
-  "avl (MKT x l r h) = ((height l = height r \<or> height l = 1 + height r \<or> height r = 1+height l) \<and> 
+| "avl (MKT x l r h) = ((height l = height r \<or> height l = 1 + height r \<or> height r = 1+height l) \<and> 
   h = max (height l) (height r) + 1 \<and> avl l \<and> avl r)"
 (*
 code_pred [inductify] avl .