src/ZF/Inductive.thy
author paulson
Sat, 29 Jun 2002 21:33:06 +0200
changeset 13259 01fa0c8dbc92
parent 12372 cd3a09c7dac9
child 13356 c9cfe1638bf2
permissions -rw-r--r--
conversion of many files to Isar format

(*  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 + QPair
  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