src/HOL/Product_Type.thy
changeset 37704 c6161bee8486
parent 37678 0040bafffdef
child 37751 89e16802b6cc
--- a/src/HOL/Product_Type.thy	Sat Jul 03 00:49:12 2010 +0200
+++ b/src/HOL/Product_Type.thy	Sat Jul 03 00:50:35 2010 +0200
@@ -158,6 +158,8 @@
     by (simp add: Pair_def Abs_prod_inject)
 qed
 
+declare prod.simps(2) [nitpick_simp del]
+
 declare weak_case_cong [cong del]
 
 
@@ -391,7 +393,7 @@
 code_const fst and snd
   (Haskell "fst" and "snd")
 
-lemma prod_case_unfold: "prod_case = (%c p. c (fst p) (snd p))"
+lemma prod_case_unfold [nitpick_def]: "prod_case = (%c p. c (fst p) (snd p))"
   by (simp add: expand_fun_eq split: prod.split)
 
 lemma fst_eqD: "fst (x, y) = a ==> x = a"