src/Doc/Tutorial/ToyList/ToyList_Test.thy
author wenzelm
Mon, 27 Oct 2014 16:11:24 +0100
changeset 58791 00916b0dd596
parent 58372 bfd497f2f4c2
child 58856 4fced55fc5b7
permissions -rw-r--r--
clarified ISABELLE_JDK_HOME vs. JAVA_HOME;

theory ToyList_Test
imports BNF_Least_Fixpoint
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