src/Doc/IsarImplementation/Base.thy
author wenzelm
Wed, 22 Jan 2014 17:02:05 +0100
changeset 55112 b1a5d603fd12
parent 48985 5386df44a037
child 56059 2390391584c2
permissions -rw-r--r--
prefer rail cartouche -- avoid back-slashed quotes; proper documentation of \<newline> syntax;

theory Base
imports Main
begin

ML_file "../antiquote_setup.ML"
setup {* Antiquote_Setup.setup *}

end