author | clasohm |
Sat, 09 Dec 1995 13:36:11 +0100 | |
changeset 1401 | 0c439768f45c |
parent 753 | ec86863e87c8 |
child 1478 | 2b8c2a7547ab |
permissions | -rw-r--r-- |
(* Title: ZF/univ.thy ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1993 University of Cambridge A small universe for lazy recursive types *) QUniv = Univ + QPair + "mono" + "equalities" + consts quniv :: i=>i defs quniv_def "quniv(A) == Pow(univ(eclose(A)))" end