| author | paulson | 
| Mon, 28 Dec 1998 16:46:15 +0100 | |
| changeset 6035 | c041fc54ab4c | 
| parent 2870 | 6d6fd10a9fdc | 
| child 6053 | 8a1059aa01f0 | 
| permissions | -rw-r--r-- | 
| 2870 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 1 | (* Title: ZF/Datatype | 
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 2 | ID: $Id$ | 
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
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: 
809diff
changeset | 4 | Copyright 1997 University of Cambridge | 
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 5 | |
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 6 | Dummy theory: brings in all ancestors needed for (Co)Datatype Declarations | 
| 124 | 7 | |
| 2870 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 8 | "Datatype" must be capital to avoid conflicts with ML's "datatype" | 
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 9 | *) | 
| 516 | 10 | |
| 2870 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 11 | Datatype = "constructor" + Inductive + Univ + QUniv + | 
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 12 | |
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 13 | end | 
| 
6d6fd10a9fdc
Now a non-trivial theory so that require_thy can find it
 paulson parents: 
809diff
changeset | 14 |