src/HOL/Predicate.thy
changeset 62390 842917225d56
parent 62026 ea3b1b0413b4
child 66012 59bf29d2b3a1
--- a/src/HOL/Predicate.thy	Tue Feb 23 15:37:18 2016 +0100
+++ b/src/HOL/Predicate.thy	Tue Feb 23 16:25:08 2016 +0100
@@ -346,11 +346,11 @@
 
 lemma not_predE: "eval (not_pred (Pred (\<lambda>u. P))) x \<Longrightarrow> (\<not> P \<Longrightarrow> thesis) \<Longrightarrow> thesis"
   unfolding not_pred_eq
-  by (auto split: split_if_asm elim: botE)
+  by (auto split: if_split_asm elim: botE)
 
 lemma not_predE': "eval (not_pred P) x \<Longrightarrow> (\<not> eval P x \<Longrightarrow> thesis) \<Longrightarrow> thesis"
   unfolding not_pred_eq
-  by (auto split: split_if_asm elim: botE)
+  by (auto split: if_split_asm elim: botE)
 lemma "f () = False \<or> f () = True"
 by simp