src/FOL/IFOL.thy
changeset 28856 5e009a80fe6d
parent 28699 32b6a8f12c1c
child 30160 5f7b17941730
child 30240 5b25fee0362c
--- a/src/FOL/IFOL.thy	Wed Nov 19 18:15:31 2008 +0100
+++ b/src/FOL/IFOL.thy	Thu Nov 20 00:03:47 2008 +0100
@@ -698,11 +698,9 @@
   then show "A == B" by (rule iff_reflection)
 qed
 
-lemma atomize_conj [atomize]:
-  fixes meta_conjunction :: "prop => prop => prop"  (infixr "&&" 2)
-  shows "(A && B) == Trueprop (A & B)"
+lemma atomize_conj [atomize]: "(A &&& B) == Trueprop (A & B)"
 proof
-  assume conj: "A && B"
+  assume conj: "A &&& B"
   show "A & B"
   proof (rule conjI)
     from conj show A by (rule conjunctionD1)
@@ -710,7 +708,7 @@
   qed
 next
   assume conj: "A & B"
-  show "A && B"
+  show "A &&& B"
   proof -
     from conj show A ..
     from conj show B ..