src/Doc/Tutorial/ToyList/ToyList_Test.thy
changeset 58372 bfd497f2f4c2
parent 58112 8081087096ad
child 58856 4fced55fc5b7
equal deleted inserted replaced
58371:7f30ec82fe40 58372:bfd497f2f4c2
     1 theory ToyList_Test
     1 theory ToyList_Test
     2 imports Old_Datatype
     2 imports BNF_Least_Fixpoint
     3 begin
     3 begin
     4 
     4 
     5 ML {*
     5 ML {*
     6   map (File.read o Path.append (Resources.master_directory @{theory}) o Path.explode)
     6   map (File.read o Path.append (Resources.master_directory @{theory}) o Path.explode)
     7     ["ToyList1.txt", "ToyList2.txt"]
     7     ["ToyList1.txt", "ToyList2.txt"]