diff -r d1d9dee7a4bf -r 3f3e9f18f302 src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy --- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy Wed Apr 21 12:10:52 2010 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Examples.thy Wed Apr 21 12:10:52 2010 +0200 @@ -789,7 +789,6 @@ code_pred [inductify, skip_proof] case_f . thm case_fP.equation -thm case_fP.intros fun fold_map_idx where "fold_map_idx f i y [] = (y, [])" @@ -935,10 +934,10 @@ code_pred [inductify] avl . thm avl.equation*) -code_pred [random_dseq inductify] avl . -thm avl.random_dseq_equation +code_pred [new_random_dseq inductify] avl . +thm avl.new_random_dseq_equation -values [random_dseq 2, 1, 7] 5 "{t:: int tree. avl t}" +values [new_random_dseq 2, 1, 7] 5 "{t:: int tree. avl t}" fun set_of where