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