src/HOL/ex/Predicate_Compile.thy
author haftmann
Fri, 25 Sep 2009 09:50:31 +0200
changeset 32705 04ce6bb14d85
parent 32672 90f3ce5d27ae
child 33112 6672184a736b
permissions -rw-r--r--
merged
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
30374
7311a1546d85 added predicate compiler, as formally checked prototype, not as user package
haftmann
parents:
diff changeset
     1
theory Predicate_Compile
32351
haftmann
parents: 32340 32318
diff changeset
     2
imports Complex_Main RPred
32668
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     3
uses
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     4
  "../Tools/Predicate_Compile/pred_compile_aux.ML"
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     5
  "../Tools/Predicate_Compile/predicate_compile_core.ML"
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     6
  "../Tools/Predicate_Compile/pred_compile_set.ML"
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     7
  "../Tools/Predicate_Compile/pred_compile_data.ML"
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     8
  "../Tools/Predicate_Compile/pred_compile_fun.ML"
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
     9
  "../Tools/Predicate_Compile/pred_compile_pred.ML"
b2de45007537 added first prototype of the extended predicate compiler
bulwahn
parents: 32667
diff changeset
    10
  "../Tools/Predicate_Compile/predicate_compile.ML"
32672
90f3ce5d27ae added first version of quickcheck based on the predicate compiler; added a few quickcheck examples
bulwahn
parents: 32668
diff changeset
    11
  "../Tools/Predicate_Compile/pred_compile_quickcheck.ML"
30374
7311a1546d85 added predicate compiler, as formally checked prototype, not as user package
haftmann
parents:
diff changeset
    12
begin
7311a1546d85 added predicate compiler, as formally checked prototype, not as user package
haftmann
parents:
diff changeset
    13
7311a1546d85 added predicate compiler, as formally checked prototype, not as user package
haftmann
parents:
diff changeset
    14
setup {* Predicate_Compile.setup *}
32672
90f3ce5d27ae added first version of quickcheck based on the predicate compiler; added a few quickcheck examples
bulwahn
parents: 32668
diff changeset
    15
setup {* Quickcheck.add_generator ("pred_compile", Pred_Compile_Quickcheck.quickcheck) *}
30374
7311a1546d85 added predicate compiler, as formally checked prototype, not as user package
haftmann
parents:
diff changeset
    16
7311a1546d85 added predicate compiler, as formally checked prototype, not as user package
haftmann
parents:
diff changeset
    17
end