src/HOL/ex/Predicate_Compile_Quickcheck_ex.thy
changeset 33375 fd3e861f8d31
parent 33257 95186fb5653c
child 33405 5c1928d5db38
--- a/src/HOL/ex/Predicate_Compile_Quickcheck_ex.thy	Fri Oct 30 01:32:06 2009 +0100
+++ b/src/HOL/ex/Predicate_Compile_Quickcheck_ex.thy	Fri Oct 30 09:55:15 2009 +0100
@@ -32,10 +32,10 @@
 | "w \<in> S\<^isub>2 \<Longrightarrow> b # w \<in> B\<^isub>2"
 | "\<lbrakk>v \<in> B\<^isub>2; v \<in> B\<^isub>2\<rbrakk> \<Longrightarrow> a # v @ w \<in> B\<^isub>2"
 
-code_pred [inductify, rpred] S\<^isub>2 .
-thm S\<^isub>2.rpred_equation
-thm A\<^isub>2.rpred_equation
-thm B\<^isub>2.rpred_equation
+code_pred [inductify, random] S\<^isub>2 .
+thm S\<^isub>2.random_equation
+thm A\<^isub>2.random_equation
+thm B\<^isub>2.random_equation
 
 values [random] 10 "{x. S\<^isub>2 x}"