author | webertj |
Fri, 11 Mar 2005 16:08:21 +0100 | |
changeset 15603 | 27a706e3a53d |
parent 13357 | 6f54e992777e |
child 16417 | 9bc16273c2d4 |
permissions | -rw-r--r-- |
12175 | 1 |
(* Title: ZF/Inductive.thy |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1993 University of Cambridge |
|
5 |
||
6 |
*) |
|
578
efc648d29dd0
ZF/Inductive.thy,.ML: renamed from "inductive" to allow re-building without
lcp
parents:
diff
changeset
|
7 |
|
13356 | 8 |
header{*Inductive and Coinductive Definitions*} |
9 |
||
13357 | 10 |
theory Inductive = Fixedpt + QPair |
12175 | 11 |
files |
12183 | 12 |
"ind_syntax.ML" |
12175 | 13 |
"Tools/cartprod.ML" |
14 |
"Tools/ind_cases.ML" |
|
15 |
"Tools/inductive_package.ML" |
|
16 |
"Tools/induct_tacs.ML" |
|
17 |
"Tools/primrec_package.ML": |
|
18 |
||
19 |
setup IndCases.setup |
|
12208 | 20 |
setup DatatypeTactics.setup |
2870
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
805
diff
changeset
|
21 |
|
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
805
diff
changeset
|
22 |
end |