src/Pure/ProofGeneral/pgml_isabelle.ML
author wenzelm
Tue, 14 Aug 2007 23:23:06 +0200
changeset 24277 6442fde2daaa
parent 23935 2a4e42ec9a54
child 25273 189db9ef803f
permissions -rw-r--r--
added implicit type mode (cf. Type.mode); added inner syntax parsers for sort/typ (no term/prop yet); infer_types: exception TYPE => error; read_vars: Syntax.parse_typ;

(*  Title:      Pure/ProofGeneral/pgml_isabelle.ML
    ID:         $Id$
    Author:     David Aspinall

PGML print mode for common Isabelle markup.
*)

signature PGML_ISABELLE =
sig
  val pgml_mode: ('a -> 'b) -> 'a -> 'b
end

structure PgmlIsabelle : PGML_ISABELLE =
struct

(** print mode **)

val pgmlN = "PGML";
fun pgml_mode f x = PrintMode.with_modes [pgmlN] f x;

val _ = Markup.add_mode pgmlN (fn markup as (name, _) => ("", ""));

end;