changeset 911 | 95ee248b3832 |
parent 910 | b91782991dc8 |
child 998 | cfd2a42d60e3 |
--- a/Quot/Examples/IntEx.thy Thu Jan 21 11:11:22 2010 +0100 +++ b/Quot/Examples/IntEx.thy Thu Jan 21 12:03:47 2010 +0100 @@ -191,10 +191,6 @@ lemma ex1tst': "\<exists>! (x :: my_int). x = x" apply(lifting ex1tst) - -apply injection -apply (rule quot_respect(9)) -apply (rule Quotient_my_int) done lemma ho_tst: "foldl my_plus x [] = x"