doc-src/TutorialI/Advanced/WFrec.thy
changeset 10795 9e888d60d3e5
parent 10654 458068404143
child 10841 2fb8089ab6cd
equal deleted inserted replaced
10794:65d18005d802 10795:9e888d60d3e5
    77 
    77 
    78 lemma wf_id: "wf r \<Longrightarrow> wf(id r)"
    78 lemma wf_id: "wf r \<Longrightarrow> wf(id r)"
    79 by simp;
    79 by simp;
    80 
    80 
    81 text{*\noindent
    81 text{*\noindent
    82 and should have appended the following hint to our above definition:
    82 and should have appended the following hint to our definition above:
    83 \indexbold{*recdef_wf}
    83 \indexbold{*recdef_wf}
    84 *}
    84 *}
    85 (*<*)
    85 (*<*)
    86 consts g :: "nat \<Rightarrow> nat"
    86 consts g :: "nat \<Rightarrow> nat"
    87 recdef g "id(less_than)"
    87 recdef g "id(less_than)"