src/HOL/Library/SML_Quickcheck.thy
author wenzelm
Sat, 07 Aug 2010 14:45:26 +0200
changeset 38222 dac5fa0ac971
parent 37390 8781d80026fc
child 39252 8f176e575a49
permissions -rw-r--r--
replaced individual Document_Model history by all-inclusive one in Session; Document_Model: provide thy_name externally, i.e. by central Isabelle plugin; tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
33084
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     1
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     2
header {* Install quickcheck of SML code generator *}
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     3
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     4
theory SML_Quickcheck
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     5
imports Main
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     6
begin
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     7
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
     8
setup {*
37390
8781d80026fc moved inductive_codegen to place where product type is available; tuned structure name
haftmann
parents: 33771
diff changeset
     9
  Inductive_Codegen.quickcheck_setup #>
33084
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
    10
  Quickcheck.add_generator ("SML", Codegen.test_term)
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
    11
*}
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
    12
cd1579e0997a turned off old quickcheck
haftmann
parents:
diff changeset
    13
end