| author | paulson |
| Fri, 18 Feb 2000 15:33:09 +0100 | |
| changeset 8253 | 975eb12aa040 |
| parent 7717 | e7ecfa617443 |
| child 9895 | 75e55370b1ae |
| 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 |
||
|
7717
e7ecfa617443
Added attribute rulify_prems (useful for modifying premises of introduction
berghofe
parents:
7705
diff
changeset
|
10 |
setup rulify_prems_attrib_setup |
|
e7ecfa617443
Added attribute rulify_prems (useful for modifying premises of introduction
berghofe
parents:
7705
diff
changeset
|
11 |
|
| 7705 | 12 |
end |