author | paulson |
Sun, 14 Jul 2002 15:14:43 +0200 | |
changeset 13356 | c9cfe1638bf2 |
parent 13259 | 01fa0c8dbc92 |
child 13357 | 6f54e992777e |
permissions | -rw-r--r-- |
(* Title: ZF/Inductive.thy ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1993 University of Cambridge *) header{*Inductive and Coinductive Definitions*} 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 end