| author | wenzelm | 
| Fri, 21 Dec 2001 23:16:17 +0100 | |
| changeset 12587 | 3f3d2ffb5df5 | 
| parent 124 | 858ab9a9b047 | 
| 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" rules quniv_def "quniv(A) == Pow(univ(eclose(A)))" end