diff -r 0b29650e3fd8 -r d8f07b5bcfae Quot/Examples/IntEx.thy --- a/Quot/Examples/IntEx.thy Tue Dec 08 22:26:01 2009 +0100 +++ b/Quot/Examples/IntEx.thy Tue Dec 08 23:30:47 2009 +0100 @@ -321,6 +321,7 @@ lemma "map (\x. PLUS x ZERO) l = l" apply(lifting lam_tst4) -done +apply(cleaning) +sorry end