doc-src/IsarRef/Base.thy
author wenzelm
Tue, 28 Aug 2012 12:52:14 +0200
changeset 48960 17dbe95eaa2a
parent 48958 12afbf6eb7f9
permissions -rw-r--r--
missing file;

theory Base
imports Pure
begin

ML_file "../antiquote_setup.ML"
setup Antiquote_Setup.setup

end