tuned
authornipkow
Thu, 08 Feb 2018 08:59:16 +0100
changeset 67575 8563eb539e7f
parent 67573 ed0a7090167d
child 67576 b01b22f9e42e
tuned
src/HOL/Product_Type.thy
--- a/src/HOL/Product_Type.thy	Mon Feb 05 08:30:19 2018 +0100
+++ b/src/HOL/Product_Type.thy	Thu Feb 08 08:59:16 2018 +0100
@@ -446,6 +446,11 @@
   \<comment> \<open>Subsumes the old \<open>split_Pair\<close> when @{term f} is the identity function.\<close>
   by (simp add: fun_eq_iff split: prod.split)
 
+(* This looks like a sensible simp-rule but appears to do more harm than good:
+lemma case_prod_const [simp]: "(\<lambda>(_,_). c) = (\<lambda>_. c)"
+by(rule case_prod_eta)
+*)
+
 lemma case_prod_comp: "(case x of (a, b) \<Rightarrow> (f \<circ> g) a b) = f (g (fst x)) (snd x)"
   by (cases x) simp