doc-src/IsarImplementation/Thy/Base.thy
author huffman
Wed, 10 Aug 2011 16:35:50 -0700
changeset 44140 2c10c35dd4be
parent 43564 9864182c6bad
child 48891 c0eafbd55de3
permissions -rw-r--r--
remove several redundant and unused theorems about derivatives

theory Base
imports Main
uses "../../antiquote_setup.ML"
begin

setup {* Antiquote_Setup.setup *}

end