doc-src/IsarRef/Base.thy
author blanchet
Tue, 28 Aug 2012 17:17:25 +0200
changeset 48977 ae12b92c145a
parent 48958 12afbf6eb7f9
permissions -rw-r--r--
updated NEWS and CONTRIBUTORS

theory Base
imports Pure
begin

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

end