src/HOL/Complex/ex/mireif.ML
changeset 26939 1035c89b4c02
parent 26423 8408edac8f6b
child 26957 e3f04fdd994d
--- a/src/HOL/Complex/ex/mireif.ML	Sat May 17 23:53:20 2008 +0200
+++ b/src/HOL/Complex/ex/mireif.ML	Sun May 18 15:04:09 2008 +0200
@@ -34,7 +34,7 @@
       | Const("RealDef.real",_)$ (Const (@{const_name "RComplete.ceiling"},_)$ t') => Neg(Floor (Neg (num_of_term vs t')))
       | Const("RealDef.real",_) $ Const (@{const_name "Int.number_of"},_)$t' => C (HOLogic.dest_numeral t')
       | Const (@{const_name "Int.number_of"},_)$t' => C (HOLogic.dest_numeral t')
-      | _ => error ("num_of_term: unknown term " ^ Sign.string_of_term CPure.thy t);
+      | _ => error ("num_of_term: unknown term " ^ Syntax.string_of_term_global CPure.thy t);
         
 
 (* pseudo reification : term -> fm *)
@@ -58,7 +58,7 @@
         E (fm_of_term (map (fn (v, n) => (v, Suc n)) vs) p)
       | Const("All",_)$Abs(xn,xT,p) => 
         A (fm_of_term (map (fn(v, n) => (v, Suc n)) vs) p)
-      | _ => error ("fm_of_term : unknown term!" ^ Sign.string_of_term CPure.thy t);
+      | _ => error ("fm_of_term : unknown term!" ^ Syntax.string_of_term_global CPure.thy t);
 
 fun start_vs t =
     let val fs = term_frees t