src/FOL/FOL.thy
changeset 28856 5e009a80fe6d
parent 28699 32b6a8f12c1c
child 30549 d2d7874648bd
--- a/src/FOL/FOL.thy	Wed Nov 19 18:15:31 2008 +0100
+++ b/src/FOL/FOL.thy	Thu Nov 20 00:03:47 2008 +0100
@@ -346,9 +346,7 @@
 lemma induct_equal_eq: "(x == y) == Trueprop(induct_equal(x, y))"
   unfolding atomize_eq induct_equal_def .
 
-lemma induct_conj_eq:
-  fixes meta_conjunction :: "prop => prop => prop"  (infixr "&&" 2)
-  shows "(A && B) == Trueprop(induct_conj(A, B))"
+lemma induct_conj_eq: "(A &&& B) == Trueprop(induct_conj(A, B))"
   unfolding atomize_conj induct_conj_def .
 
 lemmas induct_atomize = induct_forall_eq induct_implies_eq induct_equal_eq induct_conj_eq