| author | wenzelm |
| Thu, 03 Jan 2019 20:16:42 +0100 | |
| changeset 69584 | a91e32843310 |
| parent 66453 | cc19f7ca2ed6 |
| child 69605 | a96320074298 |
| 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 |
|
|
66453
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
62390
diff
changeset
|
7 |
theory Compute_Oracle imports HOL.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 |
||
| 62390 | 19 |
end |