src/Pure/ProofGeneral/pgml_isabelle.ML
author chaieb
Sat, 20 Oct 2007 12:09:30 +0200
changeset 25111 d52a58b51f1f
parent 23935 2a4e42ec9a54
child 25273 189db9ef803f
permissions -rw-r--r--
neq0_conv removed from [iff] -- causes problems by simple goals with blast, auto etc...

(*  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;