| author | haftmann |
| Fri, 26 Oct 2018 08:20:45 +0000 | |
| changeset 69194 | 6d514e128a85 |
| parent 67406 | 23307fd33906 |
| child 69282 | 94fa3376ba33 |
| permissions | -rw-r--r-- |
| 53376 | 1 |
theory ToyList_Test |
|
58926
baf5a3c28f0c
proper import of Main: BNF_Least_Fixpoint does not "contain pretty much everything", especially it lacks the 'value' command, which is defined *after* theory List;
wenzelm
parents:
58856
diff
changeset
|
2 |
imports Main |
| 53376 | 3 |
begin |
4 |
||
| 67406 | 5 |
ML \<open> |
| 58856 | 6 |
let val text = |
7 |
map (File.read o Path.append (Resources.master_directory @{theory}) o Path.explode)
|
|
8 |
["ToyList1.txt", "ToyList2.txt"] |
|
9 |
|> implode |
|
|
58926
baf5a3c28f0c
proper import of Main: BNF_Least_Fixpoint does not "contain pretty much everything", especially it lacks the 'value' command, which is defined *after* theory List;
wenzelm
parents:
58856
diff
changeset
|
10 |
in Thy_Info.script_thy Position.start text @{theory} end
|
| 67406 | 11 |
\<close> |
| 53376 | 12 |
|
13 |
end |