diff -r c656222c4dc1 -r ff6b0c1087f2 src/ZF/WF.thy --- a/src/ZF/WF.thy Tue Mar 06 15:15:49 2012 +0000 +++ b/src/ZF/WF.thy Tue Mar 06 16:06:52 2012 +0000 @@ -63,7 +63,7 @@ lemma wf_on_field_imp_wf: "wf[field(r)](r) ==> wf(r)" by (unfold wf_def wf_on_def, fast) -lemma wf_iff_wf_on_field: "wf(r) <-> wf[field(r)](r)" +lemma wf_iff_wf_on_field: "wf(r) \ wf[field(r)](r)" by (blast intro: wf_imp_wf_on wf_on_field_imp_wf) lemma wf_on_subset_A: "[| wf[A](r); B<=A |] ==> wf[B](r)" @@ -245,7 +245,7 @@ apply (elim ssubst) apply (simp (no_asm_simp) add: vimage_singleton_iff restrict_def) apply (rule_tac t = "%z. H (?x,z) " in subst_context) -apply (subgoal_tac "\y\r-``{x}. \z. :f <-> :g") +apply (subgoal_tac "\y\r-``{x}. \z. :f \ :g") apply (blast dest: transD) apply (simp add: apply_iff) apply (blast dest: transD intro: sym) @@ -364,7 +364,7 @@ text{*Minimal-element characterization of well-foundedness*} lemma wf_eq_minimal: - "wf(r) <-> (\Q x. x:Q \ (\z\Q. \y. :r \ y\Q))" + "wf(r) \ (\Q x. x:Q \ (\z\Q. \y. :r \ y\Q))" by (unfold wf_def, blast) end