src/Doc/IsarImplementation/Base.thy
author wenzelm
Sat, 15 Feb 2014 16:27:58 +0100
changeset 55500 cdbbaa3074a8
parent 48985 5386df44a037
child 56059 2390391584c2
permissions -rw-r--r--
isabelle-ml mode with separate token marker; clarified ML_Lex.gap_start: end-of-input counts as single newline;

theory Base
imports Main
begin

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

end