| author | wenzelm |
| Fri, 11 Apr 2014 19:07:56 +0200 | |
| changeset 56546 | 902960859c66 |
| parent 56208 | 06cc31dff138 |
| child 57083 | 5c26000e1042 |
| permissions | -rw-r--r-- |
| 53376 | 1 |
theory ToyList_Test |
2 |
imports Datatype |
|
3 |
begin |
|
4 |
||
5 |
ML {* (* FIXME somewhat non-standard, fragile *)
|
|
6 |
let |
|
7 |
val texts = |
|
| 56208 | 8 |
map (File.read o Path.append (Resources.master_directory @{theory}) o Path.explode)
|
| 53376 | 9 |
["ToyList1", "ToyList2"]; |
10 |
val trs = Outer_Syntax.parse Position.start (implode texts); |
|
11 |
val end_state = fold (Toplevel.command_exception false) trs Toplevel.toplevel; |
|
12 |
in @{assert} (Toplevel.is_toplevel end_state) end;
|
|
13 |
*} |
|
14 |
||
15 |
end |
|
16 |