src/HOL/Subst/Setplus.thy
changeset 968 3cdaa8724175
child 1476 608483c2122a
equal deleted inserted replaced
967:bfcb53497a99 968:3cdaa8724175
       
     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