| author | paulson |
| Wed, 22 Dec 1999 17:18:03 +0100 | |
| changeset 8074 | 36a6c38e0eca |
| parent 7998 | 3d0c34795831 |
| child 11093 | 62c2e0af1d30 |
| permissions | -rw-r--r-- |
(* Experimental theory: long division of polynomials $Id$ Author: Clemens Ballarin, started 23 June 1999 *) LongDiv = PolyHomo + consts lcoeff :: "'a::ringS up => 'a" eucl_size :: 'a::ringS => nat defs lcoeff_def "lcoeff p == coeff (deg p) p" eucl_size_def "eucl_size p == if p = <0> then 0 else deg p+1" end