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