src/HOL/WF.ML
changeset 5143 b94cd208f073
parent 5132 24f992a25adc
child 5148 74919e8f221c
--- a/src/HOL/WF.ML	Tue Jul 14 13:33:12 1998 +0200
+++ b/src/HOL/WF.ML	Wed Jul 15 10:15:13 1998 +0200
@@ -93,7 +93,7 @@
  * Wellfoundedness of subsets
  *---------------------------------------------------------------------------*)
 
-Goal "!!r. [| wf(r);  p<=r |] ==> wf(p)";
+Goal "[| wf(r);  p<=r |] ==> wf(p)";
 by (full_simp_tac (simpset() addsimps [wf_eq_minimal]) 1);
 by (Fast_tac 1);
 qed "wf_subset";
@@ -164,7 +164,7 @@
 by (simp_tac (HOL_ss addsimps [expand_fun_eq]) 1);
 qed "cuts_eq";
 
-Goalw [cut_def] "!!x. (x,a):r ==> (cut f r a)(x) = f(x)";
+Goalw [cut_def] "(x,a):r ==> (cut f r a)(x) = f(x)";
 by (asm_simp_tac HOL_ss 1);
 qed "cut_apply";