diff -r 0aaeea9255f3 -r 6267ad688ea8 Quot/Examples/FSet.thy --- a/Quot/Examples/FSet.thy Tue Jan 26 14:08:47 2010 +0100 +++ b/Quot/Examples/FSet.thy Tue Jan 26 14:48:25 2010 +0100 @@ -409,12 +409,20 @@ lemma test5: "\ (x :: 'a list \ 'a list, y) \ Respects( prod_rel (op \ ===> op \) (op \ ===> op \) -). x = y" +). (op \ ===> op \) x y" sorry lemma "All (\ (x :: 'a fset \ 'a fset, y). x = y)" apply (lifting test5) +done + +lemma test6: "\ (x :: 'a list \ 'a list, y, z) \ Respects( + prod_rel (op \ ===> op \) (prod_rel (op \ ===> op \) (op \ ===> op \)) +). (op \ ===> op \) x y \ (op \ ===> op \) y z" sorry +lemma "All (\ (x :: 'a fset \ 'a fset, y, z). x = y \ y = z)" +apply (lifting test6) +done end