doc-src/IsarImplementation/Thy/Base.thy
author wenzelm
Wed, 21 Sep 2011 15:08:15 +0200
changeset 45024 77c3e74bd954
parent 43564 9864182c6bad
child 48891 c0eafbd55de3
permissions -rw-r--r--
reduced default thread stack, to increase the success rate especially on Windows (NB: the actor worker farm tends to produce 100-200 threads for big sessions);

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

setup {* Antiquote_Setup.setup *}

end