| author | wenzelm |
| Sat, 12 Jan 2002 16:37:58 +0100 | |
| changeset 12725 | 7ede865e1fe5 |
| parent 12183 | c10cea75dd56 |
| child 13328 | 703de709a64b |
| permissions | -rw-r--r-- |
| 12175 | 1 |
(* Title: ZF/Datatype.thy |
|
2870
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
809
diff
changeset
|
2 |
ID: $Id$ |
|
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
809
diff
changeset
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
809
diff
changeset
|
4 |
Copyright 1997 University of Cambridge |
|
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
809
diff
changeset
|
5 |
|
| 12175 | 6 |
(Co)Datatype Definitions for Zermelo-Fraenkel Set Theory. |
|
2870
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
809
diff
changeset
|
7 |
*) |
| 516 | 8 |
|
| 12175 | 9 |
theory Datatype = Inductive + Univ + QUniv |
| 12183 | 10 |
files |
11 |
"Tools/datatype_package.ML" |
|
12 |
"Tools/numeral_syntax.ML": (*belongs to theory Bin*) |
|
| 12175 | 13 |
|
14 |
end |