reconsider 'pretty_setmargin' as "control" command (instead of "diag") -- it is stateful and Proof General legacy;
(* Author: Clemens Ballarin, started 17 July 1997
Summary theory of the development of (not instantiated) polynomials.
*)
theory Polynomial
imports LongDiv
begin
end