doc-src/IsarImplementation/Thy/Base.thy
author wenzelm
Thu, 24 Jun 2010 14:31:01 +0200
changeset 37528 42804fb5dd92
parent 30272 2d612824e642
child 39846 cb6634eb8926
permissions -rw-r--r--
slightly more standard data merge: Symtax.merge (K true) avoids equality on abstract type Pretty.T and gracefully accepts overriding, Symtab.join prefers first entry as usual;

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

end