merged
authorpaulson
Sun, 17 Jun 2018 22:01:16 +0100
changeset 68459 0eb751466b79
parent 68457 517aa9076fc9 (diff)
parent 68458 023b353911c5 (current diff)
child 68461 8dea233d4bae
merged
--- a/src/HOL/Product_Type.thy	Sun Jun 17 22:00:43 2018 +0100
+++ b/src/HOL/Product_Type.thy	Sun Jun 17 22:01:16 2018 +0100
@@ -670,6 +670,9 @@
 lemma pair_imageI [intro]: "(a, b) \<in> A \<Longrightarrow> f a b \<in> (\<lambda>(a, b). f a b) ` A"
   by (rule image_eqI [where x = "(a, b)"]) auto
 
+lemma Collect_const_case_prod[simp]: "{(a,b). P} = (if P then UNIV else {})"
+by auto
+
 lemma The_split_eq [simp]: "(THE (x',y'). x = x' \<and> y = y') = (x, y)"
   by blast