src/ZF/Inductive.thy
author kleing
Tue, 18 Dec 2001 21:28:01 +0100
changeset 12545 7319d384d0d3
parent 12372 cd3a09c7dac9
child 13259 01fa0c8dbc92
permissions -rw-r--r--
removed preallocated heaps axiom (now in type safety invariant)

(*  Title:      ZF/Inductive.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1993  University of Cambridge

(Co)Inductive Definitions for Zermelo-Fraenkel Set Theory.
*)

theory Inductive = Fixedpt + mono
  files
    "ind_syntax.ML"
    "Tools/cartprod.ML"
    "Tools/ind_cases.ML"
    "Tools/inductive_package.ML"
    "Tools/induct_tacs.ML"
    "Tools/primrec_package.ML":

setup IndCases.setup
setup DatatypeTactics.setup


(*belongs to theory ZF*)
declare bspec [dest?]

(*belongs to theory upair*)
declare UnI1 [elim?]  UnI2 [elim?]

end