author | wenzelm |
Tue, 12 Mar 2024 15:57:25 +0100 | |
changeset 79873 | 6c19c29ddcbe |
parent 69605 | a96320074298 |
permissions | -rw-r--r-- |
63992 | 1 |
(* Title: HOL/Library/Predicate_Compile_Quickcheck.thy |
63764 | 2 |
Author: Lukas Bulwahn, TU Muenchen |
3 |
*) |
|
35953 | 4 |
|
60500 | 5 |
section \<open>A Prototype of Quickcheck based on the Predicate Compiler\<close> |
35953 | 6 |
|
7 |
theory Predicate_Compile_Quickcheck |
|
63764 | 8 |
imports Predicate_Compile_Alternative_Defs |
35953 | 9 |
begin |
10 |
||
69605 | 11 |
ML_file \<open>../Tools/Predicate_Compile/predicate_compile_quickcheck.ML\<close> |
48891 | 12 |
|
51143
0a2371e7ced3
two target language numeral types: integer and natural, as replacement for code_numeral;
haftmann
parents:
48891
diff
changeset
|
13 |
end |