| author | wenzelm |
| Wed, 29 Jun 2005 15:13:38 +0200 | |
| changeset 16608 | 4f8d7b83c7e2 |
| parent 16417 | 9bc16273c2d4 |
| child 22814 | 4cd25f1706bb |
| 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 imports Fixedpt QPair uses "ind_syntax.ML" "Tools/cartprod.ML" "Tools/ind_cases.ML" "Tools/inductive_package.ML" "Tools/induct_tacs.ML" "Tools/primrec_package.ML" begin setup IndCases.setup setup DatatypeTactics.setup end