author | wenzelm |
Tue, 01 Oct 2024 20:39:16 +0200 | |
changeset 81091 | c007e6d9941d |
parent 69597 | ff784d5a5bfb |
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 = |
69282 | 7 |
map (File.read o Path.append \<^master_dir>) [\<^path>\<open>ToyList1.txt\<close>, \<^path>\<open>ToyList2.txt\<close>] |
58856 | 8 |
|> implode |
69597 | 9 |
in Thy_Info.script_thy Position.start text \<^theory> end |
67406 | 10 |
\<close> |
53376 | 11 |
|
12 |
end |