author | Andreas Lochbihler |
Wed, 11 Feb 2015 18:39:56 +0100 | |
changeset 59527 | edaabc1ab1ed |
parent 48891 | c0eafbd55de3 |
child 62390 | 842917225d56 |
permissions | -rw-r--r-- |
47455 | 1 |
(* Title: HOL/Matrix_LP/Compute_Oracle/Compute_Oracle.thy |
23173
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
2 |
Author: Steven Obua, TU Munich |
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
3 |
|
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
4 |
Steven Obua's evaluator. |
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
5 |
*) |
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
6 |
|
37869 | 7 |
theory Compute_Oracle imports HOL |
23173
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
8 |
begin |
51179ca0c429
proper theory setup for compute oracle (based on CPure);
wenzelm
parents:
diff
changeset
|
9 |
|
48891 | 10 |
ML_file "am.ML" |
11 |
ML_file "am_compiler.ML" |
|
12 |
ML_file "am_interpreter.ML" |
|
13 |
ML_file "am_ghc.ML" |
|
14 |
ML_file "am_sml.ML" |
|
15 |
ML_file "report.ML" |
|
16 |
ML_file "compute.ML" |
|
17 |
ML_file "linker.ML" |
|
18 |
||
23663 | 19 |
end |