src/HOL/ex/Predicate_Compile_Quickcheck.thy
changeset 35953 0460ff79bb52
parent 35952 5baac0d38977
child 35954 d87d85a5d9ab
--- a/src/HOL/ex/Predicate_Compile_Quickcheck.thy	Wed Mar 24 17:40:43 2010 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,14 +0,0 @@
-(* Author: Lukas Bulwahn, TU Muenchen *)
-
-header {* A Prototype of Quickcheck based on the Predicate Compiler *}
-
-theory Predicate_Compile_Quickcheck
-imports Main Predicate_Compile_Alternative_Defs
-uses "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"
-begin
-
-setup {* Quickcheck.add_generator ("predicate_compile_wo_ff", Predicate_Compile_Quickcheck.quickcheck_compile_term false true 4) *}
-setup {* Quickcheck.add_generator ("predicate_compile_ff_fs", Predicate_Compile_Quickcheck.quickcheck_compile_term true true 4) *}
-setup {* Quickcheck.add_generator ("predicate_compile_ff_nofs", Predicate_Compile_Quickcheck.quickcheck_compile_term true false 4) *}
-
-end
\ No newline at end of file