src/ZF/UNITY/UNITYMisc.thy
author paulson
Tue, 24 Jun 2003 16:32:59 +0200
changeset 14071 373806545656
parent 14046 6616e6c53d48
child 14072 f932be305381
permissions -rw-r--r--
Converting ZF/UNITY to Isar

(*  Title:      HOL/UNITY/UNITYMisc.thy
    ID:         $Id$
    Author:     Sidi O Ehmety, Computer Laboratory
    Copyright   2001  University of Cambridge

Some miscellaneous and add-hoc set theory concepts.
*)



UNITYMisc = Main +
constdefs
  greaterThan :: [i,i]=> i
  "greaterThan(u,A) == {x:A. u<x}"
end