Quot/Examples/FSet.thy
changeset 931 0879d144aaa3
parent 918 7be9b054f672
child 940 a792bfc1be2b
--- a/Quot/Examples/FSet.thy	Tue Jan 26 09:28:32 2010 +0100
+++ b/Quot/Examples/FSet.thy	Tue Jan 26 09:54:43 2010 +0100
@@ -377,22 +377,6 @@
 apply(assumption)
 done
 
-lemma [quot_respect]:
-  "((op \<approx> ===> op \<approx> ===> op =) ===> prod_rel op \<approx> op \<approx> ===> op =) split split"
-apply(simp)
-done
-
-thm quot_preserve
-term split
-
-
-lemma [quot_preserve]:
-  shows "(((abs_fset ---> abs_fset ---> id) ---> prod_fun rep_fset rep_fset ---> id) split) = split"
-apply(simp add: expand_fun_eq)
-apply(simp add: Quotient_abs_rep[OF Quotient_fset])
-done
-
-
 lemma test: "All (\<lambda>(x::'a list, y). x = y)"
 sorry