src/HOL/Algebra/poly/PolyRing.thy
changeset 7998 3d0c34795831
child 10448 da7d0e28f746
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Algebra/poly/PolyRing.thy	Fri Nov 05 11:14:26 1999 +0100
@@ -0,0 +1,15 @@
+(*
+    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_one_not_zero,
+   up_power_def) {| rtac refl 1 |}
+
+end