author | nipkow |
Sun, 25 Jan 2004 00:42:22 +0100 | |
changeset 14360 | e654599b114e |
parent 13735 | 7de9342aca7a |
child 14723 | b77ce15b625a |
permissions | -rw-r--r-- |
(* Experimental theory: long division of polynomials $Id$ Author: Clemens Ballarin, started 23 June 1999 *) LongDiv = PolyHomo + consts lcoeff :: "'a::ring up => 'a" eucl_size :: 'a::ring => nat defs lcoeff_def "lcoeff p == coeff p (deg p)" eucl_size_def "eucl_size p == if p = 0 then 0 else deg p+1" end