src/HOL/Library/comm_ring.ML
changeset 29265 5b4247055bd7
parent 26939 1035c89b4c02
child 30510 4120fc59dd85
--- a/src/HOL/Library/comm_ring.ML	Wed Dec 31 00:08:11 2008 +0100
+++ b/src/HOL/Library/comm_ring.ML	Wed Dec 31 00:08:13 2008 +0100
@@ -1,5 +1,4 @@
-(*  ID:         $Id$
-    Author:     Amine Chaieb
+(*  Author:     Amine Chaieb
 
 Tactic for solving equalities over commutative rings.
 *)
@@ -71,7 +70,7 @@
 fun reif_eq thy (eq as Const("op =", Type("fun", [T, _])) $ lhs $ rhs) =
       if Sign.of_sort thy (T, cr_sort) then
         let
-          val fs = term_frees eq;
+          val fs = OldTerm.term_frees eq;
           val cvs = cterm_of thy (HOLogic.mk_list T fs);
           val clhs = cterm_of thy (reif_polex T fs lhs);
           val crhs = cterm_of thy (reif_polex T fs rhs);