author | obua |
Sun, 09 May 2004 23:04:36 +0200 | |
changeset 14722 | 8e739a6eaf11 |
parent 13735 | 7de9342aca7a |
child 14723 | b77ce15b625a |
permissions | -rw-r--r-- |
7998 | 1 |
(* |
2 |
Experimental theory: long division of polynomials |
|
3 |
$Id$ |
|
4 |
Author: Clemens Ballarin, started 23 June 1999 |
|
5 |
*) |
|
6 |
||
7 |
LongDiv = PolyHomo + |
|
8 |
||
9 |
consts |
|
13735 | 10 |
lcoeff :: "'a::ring up => 'a" |
11 |
eucl_size :: 'a::ring => nat |
|
7998 | 12 |
|
13 |
defs |
|
13735 | 14 |
lcoeff_def "lcoeff p == coeff p (deg p)" |
11093 | 15 |
eucl_size_def "eucl_size p == if p = 0 then 0 else deg p+1" |
7998 | 16 |
|
17 |
end |
|
18 |