| author | nipkow | 
| Wed, 06 Nov 2002 14:02:18 +0100 | |
| changeset 13697 | e4db4f06cec1 | 
| parent 11093 | 62c2e0af1d30 | 
| permissions | -rw-r--r-- | 
| 7998 | 1 | (* | 
| 2 | Instantiate polynomials to form a ring and prove further properties | |
| 3 | $Id$ | |
| 4 | Author: Clemens Ballarin, started 20 January 1997 | |
| 5 | *) | |
| 6 | ||
| 7 | PolyRing = UnivPoly + | |
| 8 | ||
| 9 | instance | |
| 10 | up :: (ring) ring | |
| 11 | (up_a_assoc, up_l_zero, up_l_neg, up_a_comm, | |
| 11093 | 12 | up_m_assoc, up_l_one, up_l_distr, up_m_comm, | 
| 10448 | 13 |    up_inverse_def, up_divide_def, up_power_def) {| ALLGOALS (rtac refl) |}
 | 
| 7998 | 14 | |
| 15 | end |