src/Pure/primitive_defs.ML
changeset 24981 4ec3f95190bf
parent 24259 c9e05c49d02c
child 29580 117b88da143c
--- a/src/Pure/primitive_defs.ML	Thu Oct 11 19:10:22 2007 +0200
+++ b/src/Pure/primitive_defs.ML	Thu Oct 11 19:10:23 2007 +0200
@@ -7,7 +7,7 @@
 
 signature PRIMITIVE_DEFS =
 sig
-  val dest_def: Pretty.pp -> (term -> bool) -> (string -> bool) -> (string -> bool) ->
+  val dest_def: Proof.context -> (term -> bool) -> (string -> bool) -> (string -> bool) ->
     term -> (term * term) * term
   val abs_def: term -> term * term
   val mk_defpair: term * term -> string * term
@@ -22,15 +22,15 @@
   | term_kind _ = "";
 
 (*c x == t[x] to !!x. c x == t[x]*)
-fun dest_def pp check_head is_fixed is_fixedT eq =
+fun dest_def ctxt check_head is_fixed is_fixedT eq =
   let
     fun err msg = raise TERM (msg, [eq]);
     val eq_vars = Term.strip_all_vars eq;
     val eq_body = Term.strip_all_body eq;
 
     val display_terms =
-      commas_quote o map (Pretty.string_of_term pp o Syntax.bound_vars eq_vars);
-    val display_types = commas_quote o map (Pretty.string_of_typ pp);
+      commas_quote o map (Syntax.string_of_term ctxt o Syntax.bound_vars eq_vars);
+    val display_types = commas_quote o map (Syntax.string_of_typ ctxt);
 
     val (raw_lhs, rhs) = Logic.dest_equals eq_body handle TERM _ => err "Not a meta-equality (==)";
     val lhs = Envir.beta_eta_contract raw_lhs;