src/HOL/Algebra/poly/Degree.thy
author paulson
Mon, 05 Mar 2001 15:25:11 +0100
changeset 11193 851c90b23a9e
parent 7998 3d0c34795831
permissions -rw-r--r--
reorganization of HOL/UNITY, moving examples to subdirectories Simple and Comp

(*
    Degree of polynomials
    $Id$
    written by Clemens Ballarin, started 22. 1. 1997
*)

Degree = PolyRing +

consts
  deg		:: ('a::ringS) up => nat

defs
  deg_def	"deg p == LEAST n. bound n (Rep_UP p)"

end