reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp
(* Prepearing definitions for polynomials $Id$ Author: Clemens Ballarin, started 9 December 1996*)ProtoPoly = Abstract +consts bound :: [nat, nat => 'a::ringS] => booldefs bound_def "bound n f == ALL i. n<i --> f i = 0"end