src/Doc/Tutorial/ToyList/ToyList_Test.thy
author wenzelm
Wed, 25 Mar 2015 11:39:52 +0100
changeset 59809 87641097d0f3
parent 58926 baf5a3c28f0c
child 67406 23307fd33906
permissions -rw-r--r--
tuned signature;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
53376
1d4a46f1fced more robust ToyList_Test;
wenzelm
parents:
diff changeset
     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
1d4a46f1fced more robust ToyList_Test;
wenzelm
parents:
diff changeset
     3
begin
1d4a46f1fced more robust ToyList_Test;
wenzelm
parents:
diff changeset
     4
57626
2288a6f17930 more official Thy_Info.script_thy;
wenzelm
parents: 57083
diff changeset
     5
ML {*
58856
4fced55fc5b7 provide explicit theory (amending 621c052789b4);
wenzelm
parents: 58372
diff changeset
     6
  let val text =
4fced55fc5b7 provide explicit theory (amending 621c052789b4);
wenzelm
parents: 58372
diff changeset
     7
    map (File.read o Path.append (Resources.master_directory @{theory}) o Path.explode)
4fced55fc5b7 provide explicit theory (amending 621c052789b4);
wenzelm
parents: 58372
diff changeset
     8
      ["ToyList1.txt", "ToyList2.txt"]
4fced55fc5b7 provide explicit theory (amending 621c052789b4);
wenzelm
parents: 58372
diff changeset
     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
53376
1d4a46f1fced more robust ToyList_Test;
wenzelm
parents:
diff changeset
    11
*}
1d4a46f1fced more robust ToyList_Test;
wenzelm
parents:
diff changeset
    12
1d4a46f1fced more robust ToyList_Test;
wenzelm
parents:
diff changeset
    13
end