diff -r 6621d91d3c8a -r 240a39af9ec4 src/HOL/Fun_Def.thy --- a/src/HOL/Fun_Def.thy Sat Dec 17 15:22:13 2016 +0100 +++ b/src/HOL/Fun_Def.thy Sat Dec 17 15:22:13 2016 +0100 @@ -278,6 +278,16 @@ done +subsection \Yet another induction principle on the natural numbers\ + +lemma nat_descend_induct [case_names base descend]: + fixes P :: "nat \ bool" + assumes H1: "\k. k > n \ P k" + assumes H2: "\k. k \ n \ (\i. i > k \ P i) \ P k" + shows "P m" + using assms by induction_schema (force intro!: wf_measure [of "\k. Suc n - k"])+ + + subsection \Tool setup\ ML_file "Tools/Function/termination.ML"