discontinued Display.pretty_ctyp/cterm etc.;
authorwenzelm
Fri, 28 Aug 2009 21:15:22 +0200
changeset 32433 11661f4327bb
parent 32432 64f30bdd3ba1
child 32447 e78ec17718d0
discontinued Display.pretty_ctyp/cterm etc.;
NEWS
src/Pure/display.ML
--- a/NEWS	Fri Aug 28 21:04:03 2009 +0200
+++ b/NEWS	Fri Aug 28 21:15:22 2009 +0200
@@ -181,6 +181,10 @@
 or even Display.pretty_thm_without_context as last resort.
 INCOMPATIBILITY.
 
+* Discontinued Display.pretty_ctyp/cterm etc.  INCOMPATIBILITY, use
+Syntax.pretty_typ/term directly, preferably with proper context
+instead of global theory.
+
 
 *** System ***
 
--- a/src/Pure/display.ML	Fri Aug 28 21:04:03 2009 +0200
+++ b/src/Pure/display.ML	Fri Aug 28 21:15:22 2009 +0200
@@ -27,10 +27,6 @@
   val string_of_thm_without_context: thm -> string
   val pretty_thms_aux: Proof.context -> bool -> thm list -> Pretty.T
   val pretty_thms: Proof.context -> thm list -> Pretty.T
-  val pretty_ctyp: ctyp -> Pretty.T
-  val string_of_ctyp: ctyp -> string
-  val pretty_cterm: cterm -> Pretty.T
-  val string_of_cterm: cterm -> string
   val print_syntax: theory -> unit
   val pretty_full_theory: bool -> theory -> Pretty.T list
 end;
@@ -119,15 +115,6 @@
 fun pretty_thms ctxt = pretty_thms_aux ctxt true;
 
 
-(* other printing commands *)
-
-fun pretty_ctyp cT = Syntax.pretty_typ_global (Thm.theory_of_ctyp cT) (Thm.typ_of cT);
-fun string_of_ctyp cT = Syntax.string_of_typ_global (Thm.theory_of_ctyp cT) (Thm.typ_of cT);
-
-fun pretty_cterm ct = Syntax.pretty_term_global (Thm.theory_of_cterm ct) (Thm.term_of ct);
-fun string_of_cterm ct = Syntax.string_of_term_global (Thm.theory_of_cterm ct) (Thm.term_of ct);
-
-
 
 (** print theory **)