src/HOL/ex/SVC_Oracle.thy
changeset 35084 e25eedfc15ce
parent 34974 18b41bba42b5
child 35092 cfe605c54e50
--- a/src/HOL/ex/SVC_Oracle.thy	Wed Feb 10 08:49:26 2010 +0100
+++ b/src/HOL/ex/SVC_Oracle.thy	Wed Feb 10 08:49:26 2010 +0100
@@ -65,7 +65,7 @@
     (*abstraction of a real/rational expression*)
     fun rat ((c as Const(@{const_name Algebras.plus}, _)) $ x $ y) = c $ (rat x) $ (rat y)
       | rat ((c as Const(@{const_name Algebras.minus}, _)) $ x $ y) = c $ (rat x) $ (rat y)
-      | rat ((c as Const(@{const_name Algebras.divide}, _)) $ x $ y) = c $ (rat x) $ (rat y)
+      | rat ((c as Const(@{const_name Rings.divide}, _)) $ x $ y) = c $ (rat x) $ (rat y)
       | rat ((c as Const(@{const_name Algebras.times}, _)) $ x $ y) = c $ (rat x) $ (rat y)
       | rat ((c as Const(@{const_name Algebras.uminus}, _)) $ x) = c $ (rat x)
       | rat t = lit t