replaced (outdated) comments by explicit statements
authorkrauss
Mon, 26 Oct 2009 23:26:18 +0100
changeset 33215 6fd85372981e
parent 33214 885e1b7ecb33
child 33216 7c61bc5d7310
replaced (outdated) comments by explicit statements
src/HOL/Wellfounded.thy
--- a/src/HOL/Wellfounded.thy	Mon Oct 26 20:45:24 2009 +0100
+++ b/src/HOL/Wellfounded.thy	Mon Oct 26 23:26:18 2009 +0100
@@ -59,14 +59,16 @@
 lemma wf_not_sym: "wf r ==> (a, x) : r ==> (x, a) ~: r"
   by (induct a arbitrary: x set: wf) blast
 
-(* [| wf r;  ~Z ==> (a,x) : r;  (x,a) ~: r ==> Z |] ==> Z *)
-lemmas wf_asym = wf_not_sym [elim_format]
+lemma wf_asym:
+  assumes "wf r" "(a, x) \<in> r"
+  obtains "(x, a) \<notin> r"
+  by (drule wf_not_sym[OF assms])
 
 lemma wf_not_refl [simp]: "wf r ==> (a, a) ~: r"
   by (blast elim: wf_asym)
 
-(* [| wf r;  (a,a) ~: r ==> PROP W |] ==> PROP W *)
-lemmas wf_irrefl = wf_not_refl [elim_format]
+lemma wf_irrefl: assumes "wf r" obtains "(a, a) \<notin> r"
+by (drule wf_not_refl[OF assms])
 
 lemma wf_wellorderI:
   assumes wf: "wf {(x::'a::ord, y). x < y}"