src/HOL/Library/Quotient_List.thy
changeset 51377 7da251a6c16e
parent 47982 7aa35601ff65
child 51956 a4d81cdebf8b
--- a/src/HOL/Library/Quotient_List.thy	Fri Mar 08 13:21:45 2013 +0100
+++ b/src/HOL/Library/Quotient_List.thy	Fri Mar 08 13:21:52 2013 +0100
@@ -22,7 +22,12 @@
     by (induct xs ys rule: list_induct2') simp_all
 qed
 
-lemma list_all2_OO: "list_all2 (A OO B) = list_all2 A OO list_all2 B"
+lemma list_all2_mono[relator_mono]:
+  assumes "A \<le> B"
+  shows "(list_all2 A) \<le> (list_all2 B)"
+using assms by (auto intro: list_all2_mono)
+
+lemma list_all2_OO[relator_distr]: "list_all2 A OO list_all2 B = list_all2 (A OO B)"
 proof (intro ext iffI)
   fix xs ys
   assume "list_all2 (A OO B) xs ys"