src/HOL/subset.thy
author paulson
Fri, 12 May 2000 15:05:02 +0200
changeset 8862 78643f8449c6
parent 7717 e7ecfa617443
child 9895 75e55370b1ae
permissions -rw-r--r--
NatSimprocs is now a theory, not a file

(*  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