src/HOL/Algebra/poly/Polynomial.thy
author haftmann
Tue, 10 Aug 2010 15:38:33 +0200
changeset 38318 1fade69519ab
parent 35849 b5522b51cb1e
permissions -rw-r--r--
different foundations for different targets; simplified syntax handling of abbreviations

(*  Author: Clemens Ballarin, started 17 July 1997

Summary theory of the development of (not instantiated) polynomials.
*)

theory Polynomial
imports LongDiv
begin

end