src/HOL/ex/Predicate_Compile_Quickcheck.thy
author boehmes
Fri, 13 Nov 2009 15:02:51 +0100
changeset 33660 11574d52169d
parent 33250 5c2af18a3237
child 34948 2d5f2a9f7601
permissions -rw-r--r--
extended theory simpset to simplify non-linear problems

(* Author: Lukas Bulwahn, TU Muenchen *)

header {* A Prototype of Quickcheck based on the Predicate Compiler *}

theory Predicate_Compile_Quickcheck
imports Main
uses "../Tools/Predicate_Compile/predicate_compile_quickcheck.ML"
begin

setup {* Quickcheck.add_generator ("predicate_compile", Predicate_Compile_Quickcheck.quickcheck) *}

end