doc-src/TutorialI/Misc/AdvancedInd.thy
changeset 10654 458068404143
parent 10420 ef006735bee8
child 10885 90695f46440b
equal deleted inserted replaced
10653:55f33da63366 10654:458068404143
   288 Finally we should remind the reader that HOL already provides the mother of
   288 Finally we should remind the reader that HOL already provides the mother of
   289 all inductions, well-founded induction (see \S\ref{sec:Well-founded}).  For
   289 all inductions, well-founded induction (see \S\ref{sec:Well-founded}).  For
   290 example theorem @{thm[source]nat_less_induct} can be viewed (and derived) as
   290 example theorem @{thm[source]nat_less_induct} can be viewed (and derived) as
   291 a special case of @{thm[source]wf_induct} where @{term r} is @{text"<"} on
   291 a special case of @{thm[source]wf_induct} where @{term r} is @{text"<"} on
   292 @{typ nat}. The details can be found in the HOL library.
   292 @{typ nat}. The details can be found in the HOL library.
   293 *};
   293 *}
   294 
   294 (*<*)end(*>*)
   295 (*<*)
       
   296 end
       
   297 (*>*)