renamed raw to escape;
simplified pretty token metric: type int;
simplified print_mode setup: output_width and escape;
moved pretty setup to pretty.ML;
(* 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