author | wenzelm |
Sun, 17 Sep 2000 22:25:18 +0200 | |
changeset 10012 | 4961c73b5f60 |
parent 9895 | 75e55370b1ae |
child 10276 | 75e2c6cb4153 |
permissions | -rw-r--r-- |
1475 | 1 |
(* Title: HOL/subset.thy |
923 | 2 |
ID: $Id$ |
1475 | 3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
923 | 4 |
Copyright 1994 University of Cambridge |
5 |
*) |
|
6 |
||
7705 | 7 |
theory subset = Set |
8 |
files "Tools/typedef_package.ML": |
|
9 |
||
9895 | 10 |
(*belongs to theory Ord*) |
11 |
theorems linorder_cases [case_names less equal greater] = |
|
12 |
linorder_less_split |
|
13 |
||
14 |
(*belongs to theory Set*) |
|
15 |
setup Rulify.setup |
|
7717
e7ecfa617443
Added attribute rulify_prems (useful for modifying premises of introduction
berghofe
parents:
7705
diff
changeset
|
16 |
|
7705 | 17 |
end |