doc-src/IsarImplementation/Thy/base.thy
author berghofe
Fri, 07 Apr 2006 11:17:44 +0200
changeset 19357 dade85a75c9f
parent 18537 2681f9e34390
child 21374 27ae6bc4102a
permissions -rw-r--r--
Added alternative version of thms_of_proof that does not recursively descend into proofs of (named) theorems.


(* $Id$ *)

theory base
imports CPure
uses "setup.ML"
begin

end