changed "." to "$" and Cons to infix "#" to eliminate ambiguity
(* Title: Substitutions/setplus.thy Author: Martin Coen, Cambridge University Computer Laboratory Copyright 1993 University of CambridgeMinor additions to HOL's set theory*)Setplus = Set + rules ssubset_def "A < B == A <= B & ~ A=B"end