| author | wenzelm | 
| Mon, 30 May 2016 20:58:16 +0200 | |
| changeset 63183 | 4d04e14d7ab8 | 
| parent 60500 | 903bb1495239 | 
| child 63764 | f3ad26c4b2d9 | 
| permissions | -rw-r--r-- | 
| 35953 | 1  | 
(* Author: Lukas Bulwahn, TU Muenchen *)  | 
2  | 
||
| 60500 | 3  | 
section \<open>A Prototype of Quickcheck based on the Predicate Compiler\<close>  | 
| 35953 | 4  | 
|
5  | 
theory Predicate_Compile_Quickcheck  | 
|
6  | 
imports Main Predicate_Compile_Alternative_Defs  | 
|
7  | 
begin  | 
|
8  | 
||
| 48891 | 9  | 
ML_file "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"  | 
10  | 
||
| 
51143
 
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
 
haftmann 
parents: 
48891 
diff
changeset
 | 
11  | 
end  |