changeset 28290 | 4cc2b6046258 |
parent 26957 | e3f04fdd994d |
child 30161 | c26e515f1c29 |
28289:efd53393412b | 28290:4cc2b6046258 |
---|---|
7 |
7 |
8 theory Compute_Oracle imports Pure |
8 theory Compute_Oracle imports Pure |
9 uses "am.ML" "am_compiler.ML" "am_interpreter.ML" "am_ghc.ML" "am_sml.ML" "report.ML" "compute.ML" "linker.ML" |
9 uses "am.ML" "am_compiler.ML" "am_interpreter.ML" "am_ghc.ML" "am_sml.ML" "report.ML" "compute.ML" "linker.ML" |
10 begin |
10 begin |
11 |
11 |
12 setup {* Compute.setup_compute *} |
|
13 |
|
14 end |
12 end |