src/HOL/Tools/lin_arith.ML
changeset 44064 5bce8ff0d9ae
parent 43609 20760e3608fa
child 44654 d80fe56788a5
--- a/src/HOL/Tools/lin_arith.ML	Mon Aug 08 08:55:49 2011 -0700
+++ b/src/HOL/Tools/lin_arith.ML	Mon Aug 08 09:52:09 2011 -0700
@@ -151,7 +151,7 @@
               (SOME t', m'') => (SOME (mC $ s' $ t'), m'')
             | (NONE,    m'') => (SOME s', m''))
         | (NONE,    m') => demult (t, m')))
-    | demult ((mC as Const (@{const_name Rings.divide}, _)) $ s $ t, m) =
+    | demult ((mC as Const (@{const_name Fields.divide}, _)) $ s $ t, m) =
       (* FIXME: Shouldn't we simplify nested quotients, e.g. '(s/t)/u' could
          become 's/(t*u)', and '(s*t)/u' could become 's*(t/u)' ?   Note that
          if we choose to do so here, the simpset used by arith must be able to
@@ -213,7 +213,7 @@
         (case demult inj_consts (all, m) of
            (NONE,   m') => (p, Rat.add i m')
          | (SOME u, m') => add_atom u m' pi)
-    | poly (all as Const (@{const_name Rings.divide}, _) $ _ $ _, m, pi as (p, i)) =
+    | poly (all as Const (@{const_name Fields.divide}, _) $ _ $ _, m, pi as (p, i)) =
         (case demult inj_consts (all, m) of
            (NONE,   m') => (p, Rat.add i m')
          | (SOME u, m') => add_atom u m' pi)