src/HOL/subset.thy
author wenzelm
Fri, 06 Oct 2000 17:35:58 +0200
changeset 10168 50be659d4222
parent 9895 75e55370b1ae
child 10276 75e2c6cb4153
permissions -rw-r--r--
final tuning;

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

(*belongs to theory Ord*)
theorems linorder_cases [case_names less equal greater] =
  linorder_less_split

(*belongs to theory Set*)
setup Rulify.setup

end