diff -r b379ee2cddb1 -r 1413c62db675 src/HOL/ex/Predicate_Compile_ex.thy --- a/src/HOL/ex/Predicate_Compile_ex.thy Sat Oct 24 16:55:42 2009 +0200 +++ b/src/HOL/ex/Predicate_Compile_ex.thy Sat Oct 24 16:55:42 2009 +0200 @@ -446,7 +446,7 @@ code_pred (inductify_all) S\<^isub>1p . thm S\<^isub>1p.equation -(* + theorem S\<^isub>1_sound: "w \ S\<^isub>1 \ length [x \ w. x = a] = length [x \ w. x = b]" quickcheck[generator=pred_compile] @@ -477,9 +477,8 @@ | "w \ S\<^isub>3 \ b # w \ B\<^isub>3" | "\v \ B\<^isub>3; w \ B\<^isub>3\ \ a # v @ w \ B\<^isub>3" -(* code_pred (inductify_all) S\<^isub>3 . -*) + theorem S\<^isub>3_sound: "w \ S\<^isub>3 \ length [x \ w. x = a] = length [x \ w. x = b]" quickcheck[generator=pred_compile, size=10, iterations=1] @@ -488,7 +487,7 @@ lemma "\ (length w > 2) \ \ (length [x \ w. x = a] = length [x \ w. x = b])" quickcheck[size=10, generator = pred_compile] oops -*) + inductive test where "length [x \ w. x = a] = length [x \ w. x = b] ==> test w"