doc-src/IsarImplementation/Thy/base.thy
author wenzelm
Thu, 23 Oct 2008 13:52:27 +0200
changeset 28671 ed6681dd35d8
parent 26957 e3f04fdd994d
permissions -rw-r--r--
thread-safe version, with non-critical evaluation; do not re-evaluate failed result; misc tuning;


(* $Id$ *)

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

end