src/HOL/subset.thy
author oheimb
Fri, 28 Jan 2000 11:22:02 +0100
changeset 8148 5ef0b624aadb
parent 7717 e7ecfa617443
child 9895 75e55370b1ae
permissions -rw-r--r--
beautified spacing for binders with symbols syntax, analogous to HOL.thy

(*  Title:      HOL/subset.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1994  University of Cambridge
*)

theory subset = Set
files "Tools/typedef_package.ML":

setup rulify_prems_attrib_setup

end