| author | huffman | 
| Tue, 13 Dec 2011 14:02:02 +0100 | |
| changeset 45853 | cbb6f2243b52 | 
| parent 45450 | dc2236b19a3d | 
| child 48891 | c0eafbd55de3 | 
| permissions | -rw-r--r-- | 
| 35953 | 1  | 
(* Author: Lukas Bulwahn, TU Muenchen *)  | 
2  | 
||
3  | 
header {* A Prototype of Quickcheck based on the Predicate Compiler *}
 | 
|
4  | 
||
5  | 
theory Predicate_Compile_Quickcheck  | 
|
6  | 
imports Main Predicate_Compile_Alternative_Defs  | 
|
7  | 
uses "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"  | 
|
8  | 
begin  | 
|
9  | 
||
| 
43886
 
bf068e758783
adapting quickcheck based on the analysis of the predicate compiler
 
bulwahn 
parents: 
39252 
diff
changeset
 | 
10  | 
setup {* Predicate_Compile_Quickcheck.setup *}
 | 
| 
 
bf068e758783
adapting quickcheck based on the analysis of the predicate compiler
 
bulwahn 
parents: 
39252 
diff
changeset
 | 
11  | 
|
| 35953 | 12  | 
end  |