--- a/src/HOL/Product_Type.thy Thu Feb 23 20:15:49 2012 +0100
+++ b/src/HOL/Product_Type.thy Thu Feb 23 20:15:59 2012 +0100
@@ -22,7 +22,7 @@
lemma
shows [code]: "HOL.equal False P \<longleftrightarrow> \<not> P"
and [code]: "HOL.equal True P \<longleftrightarrow> P"
- and [code]: "HOL.equal P False \<longleftrightarrow> \<not> P"
+ and [code]: "HOL.equal P False \<longleftrightarrow> \<not> P"
and [code]: "HOL.equal P True \<longleftrightarrow> P"
and [code nbe]: "HOL.equal P P \<longleftrightarrow> True"
by (simp_all add: equal)