TFL/examples/Subst/Setplus.thy
author paulson
Wed, 02 Apr 1997 15:18:21 +0200
changeset 2866 0a648ebbf6d4
parent 2113 21266526ac42
permissions -rw-r--r--
Now loads blast.ML

(*  Title:      Substitutions/setplus.thy
    Author:     Martin Coen, Cambridge University Computer Laboratory
    Copyright   1993  University of Cambridge

Minor additions to HOL's set theory
*)

Setplus = Finite + 

rules

  ssubset_def    "A < B == A <= B & ~ A=B"

end