diff -r 2c72447cdc0c -r 624af16bb6e4 Quot/Examples/FSet.thy --- a/Quot/Examples/FSet.thy Tue Jan 26 13:53:56 2010 +0100 +++ b/Quot/Examples/FSet.thy Tue Jan 26 13:58:28 2010 +0100 @@ -398,4 +398,23 @@ apply(lifting test3) done +lemma test4: "\ (x :: 'a list, y, z) \ Respects( + prod_rel (op \) (prod_rel (op \) (op \)) +). x = y \ y = z" +sorry + +lemma "All (\ (x :: 'a fset, y, z). x = y \ y = z)" +apply (lifting test4) +sorry + +lemma test5: "\ (x :: 'a list \ 'a list, y, z) \ Respects( + prod_rel (op \ ===> op \) (prod_rel (op \ ===> op \) (op \ ===> op \)) +). x = y \ y = z" +sorry + +lemma "All (\ (x :: 'a fset \ 'a fset, y, z). x = y \ y = z)" +apply (lifting test5) +sorry + + end