author | nipkow |
Mon, 13 May 2002 15:27:28 +0200 | |
changeset 13145 | 59bc43b51aa2 |
parent 11093 | 62c2e0af1d30 |
child 13735 | 7de9342aca7a |
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 |
|
10 |
lcoeff :: "'a::ringS up => 'a" |
|
11 |
eucl_size :: 'a::ringS => nat |
|
12 |
||
13 |
defs |
|
14 |
lcoeff_def "lcoeff p == coeff (deg p) p" |
|
11093 | 15 |
eucl_size_def "eucl_size p == if p = 0 then 0 else deg p+1" |
7998 | 16 |
|
17 |
end |
|
18 |