src/HOL/Library/SML_Quickcheck.thy
author wenzelm
Tue, 25 May 2010 20:28:16 +0200
changeset 37117 59cee8807c29
parent 33771 17926df64f0f
child 37390 8781d80026fc
permissions -rw-r--r--
eliminated various catch-all exception patterns, guessing at the concrete exeptions that are intended here;


header {* Install quickcheck of SML code generator *}

theory SML_Quickcheck
imports Main
begin

setup {*
  InductiveCodegen.quickcheck_setup #>
  Quickcheck.add_generator ("SML", Codegen.test_term)
*}

end