doc-src/IsarImplementation/Thy/Base.thy
author wenzelm
Mon, 25 Oct 2010 11:16:23 +0200
changeset 40110 93e7935d4cb5
parent 39866 5ec01d5acd0c
child 43564 9864182c6bad
permissions -rw-r--r--
added ML antiquotation @{assert};

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

end