src/HOL/Product_Type.thy
changeset 46556 2848e36e0348
parent 46128 53e7cc599f58
child 46557 ae926869a311
--- a/src/HOL/Product_Type.thy	Mon Feb 20 08:01:08 2012 +0100
+++ b/src/HOL/Product_Type.thy	Mon Feb 20 21:04:00 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)