src/HOL/Algebra/poly/Polynomial.thy
author blanchet
Mon, 06 Jun 2011 20:36:35 +0200
changeset 43201 0c9bf1a8e0d8
parent 35849 b5522b51cb1e
permissions -rw-r--r--
make "smart" mode of "explicit_apply" smarter, by also detecting the other kind of higher-order quantification, namely "bool"s

(*  Author: Clemens Ballarin, started 17 July 1997

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

theory Polynomial
imports LongDiv
begin

end