src/HOL/Library/Predicate_Compile_Quickcheck.thy
author wenzelm
Tue, 22 Oct 2019 20:55:13 +0200
changeset 70923 98d9b78b7f47
parent 69605 a96320074298
permissions -rw-r--r--
clarified axiom_table: uniform space (e.g. like consts), e.g. relevant for export of HOL-ex.Join_Theory;

(*  Title:      HOL/Library/Predicate_Compile_Quickcheck.thy
    Author:     Lukas Bulwahn, TU Muenchen
*)

section \<open>A Prototype of Quickcheck based on the Predicate Compiler\<close>

theory Predicate_Compile_Quickcheck
  imports Predicate_Compile_Alternative_Defs
begin

ML_file \<open>../Tools/Predicate_Compile/predicate_compile_quickcheck.ML\<close>

end