src/HOL/Algebra/poly/PolyHomo.thy
author paulson
Fri, 05 Nov 1999 11:14:26 +0100
changeset 7998 3d0c34795831
child 9279 fb4186e20148
permissions -rw-r--r--
Algebra and Polynomial theories, by Clemens Ballarin
     1 (*
     2     Universal property and evaluation homomorphism of univariate polynomials
     3     $Id$
     4     Author: Clemens Ballarin, started 15 April 1997
     5 *)
     6 
     7 PolyHomo = Degree +
     8 
     9 (* Instantiate result from Degree.ML *)
    10 
    11 instance
    12   up :: (domain) domain (up_integral)
    13 
    14 consts
    15   EVAL2	:: ('a::ringS => 'b) => 'b => 'a up => 'b::ringS
    16   EVAL	:: 'a => 'a up => 'a
    17 
    18 defs
    19   EVAL2_def	"EVAL2 phi a p == SUM (deg p) (%i. phi (coeff i p) * a ^ i)"
    20   EVAL_def	"EVAL == EVAL2 (%x. x)"
    21 
    22 end