src/HOL/Library/Quotient_Product.thy
changeset 47634 091bcd569441
parent 47624 16d433895d2e
child 47635 ebb79474262c
--- a/src/HOL/Library/Quotient_Product.thy	Fri Apr 20 15:49:45 2012 +0200
+++ b/src/HOL/Library/Quotient_Product.thy	Fri Apr 20 18:29:21 2012 +0200
@@ -93,6 +93,15 @@
 
 declare [[map prod = (prod_rel, Quotient_prod)]]
 
+definition prod_pred :: "('a \<Rightarrow> bool) \<Rightarrow> ('b \<Rightarrow> bool) \<Rightarrow> 'a \<times> 'b \<Rightarrow> bool"
+where "prod_pred R1 R2 = (\<lambda>(a, b). R1 a \<and> R2 b)"
+
+lemma prod_invariant_commute [invariant_commute]: 
+  "prod_rel (Lifting.invariant P1) (Lifting.invariant P2) = Lifting.invariant (prod_pred P1 P2)"
+  apply (simp add: fun_eq_iff prod_rel_def prod_pred_def Lifting.invariant_def) 
+  apply blast
+done
+
 subsection {* Rules for quotient package *}
 
 lemma prod_quotient [quot_thm]: