doc-src/IsarImplementation/Thy/base.thy
author wenzelm
Mon, 11 Sep 2006 21:35:19 +0200
changeset 20503 503ac4c5ef91
parent 18537 2681f9e34390
child 21374 27ae6bc4102a
permissions -rw-r--r--
induct method: renamed 'fixing' to 'arbitrary';


(* $Id$ *)

theory base
imports CPure
uses "setup.ML"
begin

end