renamed Isar/isar_output.ML to Thy/thy_output.ML;
tuned messages;
Antiquote.scan_arguments (moved from here);
moved ML context stuff to from Context to ML_Context;
(* 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