doc-src/IsarImplementation/Thy/base.thy
author wenzelm
Thu, 11 Oct 2007 16:05:53 +0200
changeset 24970 050afeec89a7
parent 21374 27ae6bc4102a
child 26957 e3f04fdd994d
permissions -rw-r--r--
renamed Syntax.XXX_mode to Syntax.mode_XXX; moved ProofContext.pp to Syntax.pp;


(* $Id$ *)

theory base
imports CPure
uses "../../antiquote_setup.ML"
begin

end