diff -r d18defacda25 -r 0c5dfd2866bb Nominal/Abs.thy --- a/Nominal/Abs.thy Wed Mar 17 08:07:25 2010 +0100 +++ b/Nominal/Abs.thy Wed Mar 17 09:18:27 2010 +0100 @@ -748,6 +748,22 @@ apply (simp add: swap_fresh_fresh) done +(* TODO: The following lemmas can be moved somewhere... *) +lemma split_rsp2[quot_respect]: "((R1 ===> R2 ===> prod_rel R1 R2 ===> op =) ===> + prod_rel R1 R2 ===> prod_rel R1 R2 ===> op =) split split" + by auto + +lemma split_prs2[quot_preserve]: + assumes q1: "Quotient R1 Abs1 Rep1" + and q2: "Quotient R2 Abs2 Rep2" + shows "((Abs1 ---> Abs2 ---> prod_fun Abs1 Abs2 ---> id) ---> prod_fun Rep1 Rep2 ---> prod_fun Rep1 Rep2 ---> id) split = split" + by (simp add: expand_fun_eq Quotient_abs_rep[OF q1] Quotient_abs_rep[OF q2]) + +lemma alpha_gen2: + "(bs, x1, x2) \gen (\(x1, y1) (x2, y2). R1 x1 x2 \ R2 y1 y2) (\(a, b). f1 a \ f2 b) pi (cs, y1, y2) = + (f1 x1 \ f2 x2 - bs = f1 y1 \ f2 y2 - cs \ (f1 x1 \ f2 x2 - bs) \* pi \ R1 (pi \ x1) y1 \ R2 (pi \ x2) y2)" +by (simp add: alpha_gen) + end