author | wenzelm |
Sun, 02 Nov 2014 17:20:45 +0100 | |
changeset 58881 | b9556a055632 |
parent 58812 | 5a9a2d3b9f8b |
child 60500 | 903bb1495239 |
permissions | -rw-r--r-- |
35953 | 1 |
(* Author: Lukas Bulwahn, TU Muenchen *) |
2 |
||
58881 | 3 |
section {* A Prototype of Quickcheck based on the Predicate Compiler *} |
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 |