src/HOL/Wellfounded.thy
changeset 44921 58eef4843641
parent 44144 74b3751ea271
child 44937 22c0857b8aab
--- a/src/HOL/Wellfounded.thy	Tue Sep 13 08:21:51 2011 -0700
+++ b/src/HOL/Wellfounded.thy	Tue Sep 13 17:07:33 2011 -0700
@@ -190,7 +190,7 @@
   "wfP (\<lambda>x y. False)"
 proof -
   have "wfP bot" by (fact wf_empty [to_pred bot_empty_eq2])
-  then show ?thesis by (simp add: bot_fun_def bot_bool_def)
+  then show ?thesis by (simp add: bot_fun_def)
 qed
 
 lemma wf_Int1: "wf r ==> wf (r Int r')"
@@ -573,7 +573,7 @@
 
 theorem accp_wfPI: "\<forall>x. accp r x ==> wfP r"
   apply (rule wfPUNIVI)
-  apply (induct_tac P x rule: accp_induct)
+  apply (rule_tac P=P in accp_induct)
    apply blast
   apply blast
   done