doc-src/IsarRef/Thy/Base.thy
author wenzelm
Tue, 28 Aug 2012 12:22:10 +0200
changeset 48956 d54a3d39ba85
parent 48891 c0eafbd55de3
permissions -rw-r--r--
prefer doc-src/pdfsetup.sty; moved IsarRef/Thy/ZF_Specific.thy to ZF/ZF_Isar.thy to avoid dependence of IsarRef on another object-logic;

theory Base
imports Pure
begin

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

end