src/ZF/upair.thy
author paulson
Fri, 11 Aug 2000 13:26:40 +0200
changeset 9577 9e66e8ed8237
parent 9570 e16e168984e1
child 9907 473a6604da94
permissions -rw-r--r--
ZF arith

(*  Title:      ZF/upair.thy
    ID:         $Id$
    Author:     Lawrence C Paulson and Martin D Coen, CU Computer Laboratory
    Copyright   1993  University of Cambridge

Dummy theory, but holds the standard ZF simpset.
*)

theory upair = ZF
files "Tools/typechk":

setup
  TypeCheck.setup

end