src/HOL/Algebra/poly/PolyRing.thy
author ballarin
Sat, 10 Feb 2001 08:52:41 +0100
changeset 11093 62c2e0af1d30
parent 10448 da7d0e28f746
permissions -rw-r--r--
Changes to HOL/Algebra: - Axclasses consolidated (axiom one_not_zero). - Now uses summation operator setsum; SUM has been removed. - Priority of infix assoc changed to 50, in accordance to dvd.

(*
    Instantiate polynomials to form a ring and prove further properties
    $Id$
    Author: Clemens Ballarin, started 20 January 1997
*)

PolyRing = UnivPoly +

instance
  up :: (ring) ring
  (up_a_assoc, up_l_zero, up_l_neg, up_a_comm, 
   up_m_assoc, up_l_one, up_l_distr, up_m_comm,
   up_inverse_def, up_divide_def, up_power_def) {| ALLGOALS (rtac refl) |}

end