src/HOL/Recdef.thy
author wenzelm
Wed, 25 Aug 1999 20:49:02 +0200
changeset 7357 d0e16da40ea2
parent 6438 e55a1869ed38
child 7701 2c8c3b7003e5
permissions -rw-r--r--
proper bootstrap of HOL theory and packages;


theory Recdef = WF_Rel
files "Tools/recdef_package.ML" "Tools/induct_method.ML":

setup RecdefPackage.setup
setup InductMethod.setup

end