tuned whitespace
authorhaftmann
Thu, 23 Feb 2012 20:15:59 +0100
changeset 46630 3abc964cdc45
parent 46629 8d3442b79f9c
child 46631 2c5c003cee35
tuned whitespace
src/HOL/Product_Type.thy
--- 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)