src/HOL/List.thy
changeset 57248 5496011859eb
parent 57243 8c261f0a9b32
parent 57247 8191ccf6a1bd
child 57308 e02fcb7e63c3
--- a/src/HOL/List.thy	Thu Jun 12 17:50:49 2014 +0200
+++ b/src/HOL/List.thy	Thu Jun 12 18:47:27 2014 +0200
@@ -2711,7 +2711,7 @@
 
 subsubsection {* @{const List.product} and @{const product_lists} *}
 
-lemma product_list_set:
+lemma set_product[simp]:
   "set (List.product xs ys) = set xs \<times> set ys"
   by (induct xs) auto
 
@@ -3332,10 +3332,8 @@
 qed (auto simp: dec_def)
 
 lemma distinct_product:
-  assumes "distinct xs" and "distinct ys"
-  shows "distinct (List.product xs ys)"
-  using assms by (induct xs)
-    (auto intro: inj_onI simp add: product_list_set distinct_map)
+  "distinct xs \<Longrightarrow> distinct ys \<Longrightarrow> distinct (List.product xs ys)"
+by (induct xs) (auto intro: inj_onI simp add: distinct_map)
 
 lemma distinct_product_lists:
   assumes "\<forall>xs \<in> set xss. distinct xs"