1
(*
2
Prepearing definitions for polynomials
3
$Id$
4
Author: Clemens Ballarin, started 9 December 1996
5
*)
6
7
ProtoPoly = Abstract +
8
9
consts
10
bound :: [nat, nat => 'a::ringS] => bool
11
12
defs
13
bound_def "bound n f == ALL i. n<i --> f i = <0>"
14
15
end