doc-src/TutorialI/Types/Setup.thy
author blanchet
Fri, 04 Dec 2009 17:19:59 +0100
changeset 33982 1ae222745c4a
parent 31678 752f23a37240
child 43564 9864182c6bad
permissions -rw-r--r--
fixed paths in Nitpick's ML file headers

theory Setup
imports Main
uses
  "../../antiquote_setup.ML"
  "../../more_antiquote.ML"
begin

end