src/HOL/Algebra/poly/UnivPoly2.thy
changeset 24993 92dfacb32053
parent 23350 50c5b0912a0c
child 25762 c03e9d04b3e4
--- a/src/HOL/Algebra/poly/UnivPoly2.thy	Fri Oct 12 08:20:45 2007 +0200
+++ b/src/HOL/Algebra/poly/UnivPoly2.thy	Fri Oct 12 08:20:46 2007 +0200
@@ -82,6 +82,7 @@
 instance up :: (plus) plus ..
 instance up :: (minus) minus ..
 instance up :: (times) times ..
+instance up :: (Divides.div) Divides.div ..
 instance up :: (inverse) inverse ..
 instance up :: (power) power ..
 
@@ -96,7 +97,7 @@
                 (* note: - 1 is different from -1; latter is of class number *)
 
   up_minus_def:   "(a::'a::{plus, minus} up) - b == a + (-b)"
-  up_inverse_def: "inverse (a::'a::{zero, one, times, inverse} up) == 
+  up_inverse_def: "inverse (a::'a::{zero, one, Divides.div, inverse} up) == 
                      (if a dvd 1 then THE x. a*x = 1 else 0)"
   up_divide_def:  "(a::'a::{times, inverse} up) / b == a * inverse b"
   up_power_def:   "(a::'a::{one, times, power} up) ^ n ==