src/HOL/HOL.thy
changeset 28699 32b6a8f12c1c
parent 28682 5de9fc98ad96
child 28741 1b257449f804
--- a/src/HOL/HOL.thy	Mon Oct 27 18:14:34 2008 +0100
+++ b/src/HOL/HOL.thy	Tue Oct 28 11:03:07 2008 +0100
@@ -846,7 +846,7 @@
 qed
 
 lemma atomize_conj [atomize]:
-  includes meta_conjunction_syntax
+  fixes meta_conjunction :: "prop => prop => prop"  (infixr "&&" 2)
   shows "(A && B) == Trueprop (A & B)"
 proof
   assume conj: "A && B"
@@ -1504,7 +1504,7 @@
   by (unfold atomize_eq induct_equal_def)
 
 lemma induct_conj_eq:
-  includes meta_conjunction_syntax
+  fixes meta_conjunction :: "prop => prop => prop"  (infixr "&&" 2)
   shows "(A && B) == Trueprop (induct_conj A B)"
   by (unfold atomize_conj induct_conj_def)