| author | wenzelm | 
| Sat, 02 Sep 2000 21:48:10 +0200 | |
| changeset 9802 | adda1dc18bb8 | 
| parent 9570 | e16e168984e1 | 
| child 9907 | 473a6604da94 | 
| permissions | -rw-r--r-- | 
| 2469 | 1 | (* Title: ZF/upair.thy | 
| 2 | ID: $Id$ | |
| 3 | Author: Lawrence C Paulson and Martin D Coen, CU Computer Laboratory | |
| 4 | Copyright 1993 University of Cambridge | |
| 5 | ||
| 2872 
ac81a17f86f8
Moved definitions (binary intersection, etc.) from upair.thy back to ZF.thy
 paulson parents: 
2469diff
changeset | 6 | Dummy theory, but holds the standard ZF simpset. | 
| 2469 | 7 | *) | 
| 8 | ||
| 9570 
e16e168984e1
installation of cancellation simprocs for the integers
 paulson parents: 
6153diff
changeset | 9 | theory upair = ZF | 
| 
e16e168984e1
installation of cancellation simprocs for the integers
 paulson parents: 
6153diff
changeset | 10 | files "Tools/typechk": | 
| 6153 | 11 | |
| 12 | setup | |
| 13 | TypeCheck.setup | |
| 14 | ||
| 15 | end | |
| 16 |