| author | mengj |
| Fri, 28 Apr 2006 05:59:32 +0200 | |
| changeset 19491 | cd6c71c57f53 |
| parent 16417 | 9bc16273c2d4 |
| child 22814 | 4cd25f1706bb |
| 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 |
|
|
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
paulson
parents:
809
diff
changeset
|
6 |
*) |
| 516 | 7 |
|
| 13328 | 8 |
header{*Datatype and CoDatatype Definitions*}
|
9 |
||
| 16417 | 10 |
theory Datatype imports Inductive Univ QUniv |
11 |
uses |
|
| 12183 | 12 |
"Tools/datatype_package.ML" |
| 16417 | 13 |
"Tools/numeral_syntax.ML" begin (*belongs to theory Bin*) |
| 12175 | 14 |
|
15 |
end |