diff -r 2848e36e0348 -r ae926869a311 src/HOL/Product_Type.thy --- a/src/HOL/Product_Type.thy Mon Feb 20 21:04:00 2012 +0100 +++ b/src/HOL/Product_Type.thy Tue Feb 21 08:15:42 2012 +0100 @@ -22,7 +22,7 @@ lemma shows [code]: "HOL.equal False P \ \ P" and [code]: "HOL.equal True P \ P" - and [code]: "HOL.equal P False \ \ P" + and [code]: "HOL.equal P False \ \ P" and [code]: "HOL.equal P True \ P" and [code nbe]: "HOL.equal P P \ True" by (simp_all add: equal)