--- a/src/HOL/HOL.thy Wed Oct 31 20:00:35 2001 +0100
+++ b/src/HOL/HOL.thy Wed Oct 31 21:58:04 2001 +0100
@@ -206,7 +206,7 @@
subsubsection {* Atomizing meta-level connectives *}
lemma atomize_all [atomize]: "(!!x. P x) == Trueprop (ALL x. P x)"
-proof (rule equal_intr_rule)
+proof
assume "!!x. P x"
show "ALL x. P x" by (rule allI)
next
@@ -215,7 +215,7 @@
qed
lemma atomize_imp [atomize]: "(A ==> B) == Trueprop (A --> B)"
-proof (rule equal_intr_rule)
+proof
assume r: "A ==> B"
show "A --> B" by (rule impI) (rule r)
next
@@ -224,7 +224,7 @@
qed
lemma atomize_eq [atomize]: "(x == y) == Trueprop (x = y)"
-proof (rule equal_intr_rule)
+proof
assume "x == y"
show "x = y" by (unfold prems) (rule refl)
next
@@ -233,7 +233,7 @@
qed
lemma atomize_conj [atomize]: "(!!C. (A ==> B ==> PROP C) ==> PROP C) == Trueprop (A & B)"
-proof (rule equal_intr_rule)
+proof
assume "!!C. (A ==> B ==> PROP C) ==> PROP C"
show "A & B" by (rule conjI)
next