src/Doc/Tutorial/ToyList/ToyList_Test.thy
author wenzelm
Fri, 15 Aug 2014 13:39:59 +0200
changeset 57975 c657c68a60ab
parent 57626 2288a6f17930
child 58112 8081087096ad
permissions -rw-r--r--
explicit system message for protocol failure -- show on Syslog panel instead of Raw Output; more robust crash recovery: warning could crash again;

theory ToyList_Test
imports Datatype
begin

ML {*
  map (File.read o Path.append (Resources.master_directory @{theory}) o Path.explode)
    ["ToyList1.txt", "ToyList2.txt"]
  |> implode
  |> Thy_Info.script_thy Position.start
*}

end