src/HOL/ex/Unification.thy
changeset 62390 842917225d56
parent 61933 cf58b5b794b2
child 67443 3abf6a722518
--- a/src/HOL/ex/Unification.thy	Tue Feb 23 15:37:18 2016 +0100
+++ b/src/HOL/ex/Unification.thy	Tue Feb 23 16:25:08 2016 +0100
@@ -285,7 +285,7 @@
       thus ?thesis by auto
     qed auto
   qed
-qed (auto split: split_if_asm)
+qed (auto split: if_split_asm)
 
 
 text \<open>The result of a unification is either the identity
@@ -458,7 +458,7 @@
       by (rule subst_eq_intro, auto simp:subst_eq_dest[OF eqv] subst_eq_dest[OF eqv2])
     thus "\<exists>\<gamma>. \<sigma>' \<doteq> \<sigma> \<lozenge> \<gamma>" ..
   qed
-qed (auto simp: MGU_Const intro: MGU_Var MGU_Var[symmetric] split: split_if_asm)
+qed (auto simp: MGU_Const intro: MGU_Var MGU_Var[symmetric] split: if_split_asm)
 
 
 subsection \<open>Unification returns Idempotent Substitution\<close>