added an intro lemma for freshness of products; set up
the simplifier so that it can deal with the compact and
long notation for freshness constraints (FIXME: it should
also be able to deal with the special case of freshness
of atoms)
(* Title: Pure/CPure.thy
ID: $Id$
The CPure theory -- Pure with alternative application syntax.
*)
theory CPure
imports Pure
begin
setup -- {* Some syntax modifications, see ROOT.ML *}
end