src/HOL/Recdef.thy
author wenzelm
Tue, 05 Oct 1999 18:16:53 +0200
changeset 7741 874abb8aa65b
parent 7701 2c8c3b7003e5
child 8303 5e7037409118
permissions -rw-r--r--
added document;

(*  Title:      HOL/Recdef.thy
    ID:         $Id$
    Author:     Konrad Slind

TFL: recursive function definitions.
*)

theory Recdef = WF_Rel + Datatype
files
  (*establish a base of common and/or helpful functions*)
  "../TFL/utils.sig"

  "../TFL/usyntax.sig"
  "../TFL/rules.sig"
  "../TFL/thry.sig"
  "../TFL/thms.sig"
  "../TFL/tfl.sig"
  "../TFL/utils.sml"

  (*supply implementations*)
  "../TFL/usyntax.sml"
  "../TFL/thms.sml"
  "../TFL/dcterm.sml"
  "../TFL/rules.sml"
  "../TFL/thry.sml"

  (*link system and specialize for Isabelle*)
  "../TFL/tfl.sml"
  "../TFL/post.sml"

  (*theory extender wrapper module*)
  "Tools/recdef_package.ML"
  "Tools/induct_method.ML":

setup RecdefPackage.setup
setup InductMethod.setup

end