src/Doc/Tutorial/Misc/simp.thy
changeset 62392 747d36865c2c
parent 48985 5386df44a037
child 67350 f061129d891b
--- a/src/Doc/Tutorial/Misc/simp.thy	Tue Feb 23 16:41:14 2016 +0100
+++ b/src/Doc/Tutorial/Misc/simp.thy	Tue Feb 23 17:47:23 2016 +0100
@@ -268,11 +268,11 @@
 The goal can be split by a special method, \methdx{split}:
 *}
 
-apply(split split_if)
+apply(split if_split)
 
 txt{*\noindent
 @{subgoals[display,indent=0]}
-where \tdx{split_if} is a theorem that expresses splitting of
+where \tdx{if_split} is a theorem that expresses splitting of
 @{text"if"}s. Because
 splitting the @{text"if"}s is usually the right proof strategy, the
 simplifier does it automatically.  Try \isacommand{apply}@{text"(simp)"}
@@ -316,7 +316,7 @@
 (*<*)
 lemma "dummy=dummy"
 (*>*)
-apply(simp split del: split_if)
+apply(simp split del: if_split)
 (*<*)
 oops
 (*>*)
@@ -334,11 +334,11 @@
 
 The split rules shown above are intended to affect only the subgoal's
 conclusion.  If you want to split an @{text"if"} or @{text"case"}-expression
-in the assumptions, you have to apply \tdx{split_if_asm} or
+in the assumptions, you have to apply \tdx{if_split_asm} or
 $t$@{text".split_asm"}: *}
 
 lemma "if xs = [] then ys \<noteq> [] else ys = [] \<Longrightarrow> xs @ ys \<noteq> []"
-apply(split split_if_asm)
+apply(split if_split_asm)
 
 txt{*\noindent
 Unlike splitting the conclusion, this step creates two