src/HOL/Library/SML_Quickcheck.thy
author wenzelm
Mon, 06 Sep 2010 14:18:16 +0200
changeset 39157 b98909faaea8
parent 37390 8781d80026fc
child 39252 8f176e575a49
permissions -rw-r--r--
more explicit HOL-Proofs sessions, including former ex/Hilbert_Classical.thy which works in parallel mode without the antiquotation option "margin" (which is still critical);


header {* Install quickcheck of SML code generator *}

theory SML_Quickcheck
imports Main
begin

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

end