src/HOL/Algebra/poly/ProtoPoly.thy
author wenzelm
Wed, 15 Mar 2000 18:22:39 +0100
changeset 8459 c32b64394963
parent 7998 3d0c34795831
child 11093 62c2e0af1d30
permissions -rw-r--r--
added pretty_goals(_marker); pretty chunks;

(*
    Prepearing definitions for polynomials
    $Id$
    Author: Clemens Ballarin, started 9 December 1996
*)

ProtoPoly = Abstract +

consts
  bound :: [nat, nat => 'a::ringS] => bool

defs
  bound_def  "bound n f == ALL i. n<i --> f i = <0>"

end