diff -r bd1354127574 -r cf7a5c863831 thys/Exercises.thy --- a/thys/Exercises.thy Fri Dec 30 23:41:44 2022 +0000 +++ b/thys/Exercises.thy Wed Feb 15 11:52:22 2023 +0000 @@ -30,7 +30,10 @@ zeroable r1 \ zeroable r2 \ (atmostempty r1 \ atmostempty r2)" | "atmostempty (STAR r) = atmostempty r" - +lemma "atmostempty r \ (zeroable r \ nullable r)" + apply(induct r) + apply(auto) + done fun somechars :: "rexp \ bool" @@ -40,8 +43,7 @@ | "somechars (CH c) \ True" | "somechars (ALT r1 r2) \ somechars r1 \ somechars r2" | "somechars (SEQ r1 r2) \ - (\ zeroable r1 \ somechars r2) \ (\ zeroable r2 \ somechars r1) \ - (somechars r1 \ nullable r2) \ (somechars r2 \ nullable r1)" + (\ zeroable r1 \ somechars r2) \ (\ zeroable r2 \ somechars r1)" | "somechars (STAR r) \ somechars r" lemma somechars_correctness: