diff -r 0140cc7b26ad -r d0b74fdd6067 src/HOL/Product_Type.thy --- a/src/HOL/Product_Type.thy Wed Dec 05 14:15:39 2007 +0100 +++ b/src/HOL/Product_Type.thy Wed Dec 05 14:15:45 2007 +0100 @@ -24,6 +24,17 @@ declare case_split [cases type: bool] -- "prefer plain propositional version" +lemma [code func]: + shows "False = P \ \ P" + and "True = P \ P" + and "P = False \ \ P" + and "P = True \ P" by simp_all + +code_const "op = \ bool \ bool \ bool" + (Haskell infixl 4 "==") + +code_instance bool :: eq + (Haskell -) subsection {* Unit *}