Nominal/Abs.thy
changeset 2447 76be909eaf04
parent 2435 3772bb3bd7ce
child 2460 16d32eddc17f
--- a/Nominal/Abs.thy	Sat Aug 28 13:41:31 2010 +0800
+++ b/Nominal/Abs.thy	Sat Aug 28 18:15:23 2010 +0800
@@ -568,16 +568,6 @@
   and   "Abs_res bs x = Abs_res cs y \<longleftrightarrow> (\<exists>p. (bs, x) \<approx>res (op =) supp p (cs, y))"
   and   "Abs_lst bsl x = Abs_lst csl y \<longleftrightarrow> (\<exists>p. (bsl, x) \<approx>lst (op =) supp p (csl, y))"
   by (lifting alphas_abs)
-
-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])
 *)