doc-src/IsarImplementation/Thy/base.thy
author blanchet
Sun, 01 Mar 2009 18:40:16 +0100
changeset 30238 d8944fd4365e
parent 26957 e3f04fdd994d
permissions -rw-r--r--
Added "nitpick_const_def" attribute, for overriding the definition axiom of a constant.


(* $Id$ *)

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

end