doc-src/TutorialI/Recdef/termination.thy
changeset 10522 ed3964d1f1a4
parent 10186 499637e8f2c6
child 10654 458068404143
equal deleted inserted replaced
10521:06206298e4d0 10522:ed3964d1f1a4
    11 from them) as theorems. For example, look (via \isacommand{thm}) at
    11 from them) as theorems. For example, look (via \isacommand{thm}) at
    12 @{thm[source]sep.simps} and @{thm[source]sep1.simps} to see that they define
    12 @{thm[source]sep.simps} and @{thm[source]sep1.simps} to see that they define
    13 the same function. What is more, those equations are automatically declared as
    13 the same function. What is more, those equations are automatically declared as
    14 simplification rules.
    14 simplification rules.
    15 
    15 
    16 In general, Isabelle may not be able to prove all termination condition
    16 In general, Isabelle may not be able to prove all termination conditions
    17 (there is one for each recursive call) automatically. For example,
    17 (there is one for each recursive call) automatically. For example,
    18 termination of the following artificial function
    18 termination of the following artificial function
    19 *}
    19 *}
    20 
    20 
    21 consts f :: "nat\<times>nat \<Rightarrow> nat";
    21 consts f :: "nat\<times>nat \<Rightarrow> nat";