diff -r dd58f13a8eb4 -r eb85850d3eb7 src/HOL/Library/Commutative_Ring.thy --- a/src/HOL/Library/Commutative_Ring.thy Fri Nov 17 02:19:55 2006 +0100 +++ b/src/HOL/Library/Commutative_Ring.thy Fri Nov 17 02:20:03 2006 +0100 @@ -48,14 +48,14 @@ text {* Create polynomial normalized polynomials given normalized inputs. *} definition - mkPinj :: "nat \ 'a pol \ 'a pol" + mkPinj :: "nat \ 'a pol \ 'a pol" where "mkPinj x P = (case P of Pc c \ Pc c | Pinj y P \ Pinj (x + y) P | PX p1 y p2 \ Pinj x P)" definition - mkPX :: "'a::{comm_ring,recpower} pol \ nat \ 'a pol \ 'a pol" + mkPX :: "'a::{comm_ring,recpower} pol \ nat \ 'a pol \ 'a pol" where "mkPX P i Q = (case P of Pc c \ (if (c = 0) then (mkPinj 1 Q) else (PX P i Q)) | Pinj j R \ PX P i Q | @@ -128,7 +128,7 @@ text {* Substraction *} definition - sub :: "'a::{comm_ring,recpower} pol \ 'a pol \ 'a pol" + sub :: "'a::{comm_ring,recpower} pol \ 'a pol \ 'a pol" where "sub p q = add (p, neg q)" text {* Square for Fast Exponentation *}