src/Doc/Tutorial/ToyList/ToyList_Test.thy
author blanchet
Wed, 03 Sep 2014 22:46:54 +0200
changeset 58163 c1e32fe387f4
parent 58112 8081087096ad
child 58372 bfd497f2f4c2
permissions -rw-r--r--
added tests for new 'countable_datatype' proof method

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