doc-src/TutorialI/Types/Setup.thy
changeset 31678 752f23a37240
child 43564 9864182c6bad
equal deleted inserted replaced
31677:799aecc0df56 31678:752f23a37240
       
     1 theory Setup
       
     2 imports Main
       
     3 uses
       
     4   "../../antiquote_setup.ML"
       
     5   "../../more_antiquote.ML"
       
     6 begin
       
     7 
       
     8 end