changeset 0 | 7949f97df77a |
-1:000000000000 | 0:7949f97df77a |
---|---|
1 (* Title: Substitutions/setplus.thy |
|
2 Author: Martin Coen, Cambridge University Computer Laboratory |
|
3 Copyright 1993 University of Cambridge |
|
4 |
|
5 Minor additions to HOL's set theory |
|
6 *) |
|
7 |
|
8 Setplus = Set + |
|
9 |
|
10 rules |
|
11 |
|
12 ssubset_def "A < B == A <= B & ~ A=B" |
|
13 |
|
14 end |