changeset 62067 | 0fd850943901 |
parent 62065 | 1546a042e87b |
child 62072 | bf3d9f113474 |
--- a/src/HOL/Library/Polynomial.thy Tue Jan 05 17:54:21 2016 +0100 +++ b/src/HOL/Library/Polynomial.thy Tue Jan 05 20:23:49 2016 +0100 @@ -2190,7 +2190,7 @@ qed -section{*lead coefficient*} +subsection {* Leading coefficient *} definition lead_coeff:: "'a::zero poly \<Rightarrow> 'a" where "lead_coeff p= coeff p (degree p)"