# HG changeset patch # User Christian Urban # Date 1515724415 0 # Node ID bfab5aded21d7abcaec69c5c9e71ad0af55a10dc # Parent 281ce101cda6d045466b38aaa6c29f9396bd3c65 updated diff -r 281ce101cda6 -r bfab5aded21d Literature/aho1990.pdf Binary file Literature/aho1990.pdf has changed diff -r 281ce101cda6 -r bfab5aded21d thys/Exercises.thy --- a/thys/Exercises.thy Thu Dec 07 12:45:22 2017 +0000 +++ b/thys/Exercises.thy Fri Jan 12 02:33:35 2018 +0000 @@ -75,6 +75,10 @@ (\ zeroable r1 \ infinitestrings r2) \ (\ zeroable r2 \ infinitestrings r1)" | "infinitestrings (STAR r) = (\ atmostempty r)" + + + + lemma Star_atmostempty: assumes "A \ {[]}" shows "A\ \ {[]}"