diff -r 9261d980225d -r 97f0221add25 thys2/SizeBound4.thy --- a/thys2/SizeBound4.thy Fri Feb 04 00:35:34 2022 +0000 +++ b/thys2/SizeBound4.thy Fri Feb 04 11:12:24 2022 +0000 @@ -1449,6 +1449,40 @@ using bsimp_ASEQ_idem apply presburger oops +lemma neg: + shows " \(\r2. r1 \ r2 \ (r2 \* bsimp r1) )" + apply(rule notI) + apply(erule exE) + apply(erule conjE) + oops + + + + +lemma reduction_always_in_bsimp: + shows " \ r1 \ r2 ; \(r2 \* bsimp r1)\ \ False" + apply(erule rrewrite.cases) + apply simp + apply auto + + oops + +(* +AALTs [] [AZERO, AALTs(bs1, [a, b]) ] +rewrite seq 1: \ AALTs [] [ AALTs(bs1, [a, b]) ] \ +fuse [] (AALTs bs1, [a, b]) +rewrite seq 2: \ AALTs [] [AZERO, (fuse bs1 a), (fuse bs1 b)]) ] + +*) + +lemma normal_bsimp: + shows "\r'. bsimp r \ r'" + oops + + (*r' size bsimp r > size r' + r' \* bsimp bsimp r +size bsimp r > size r' \ size bsimp bsimp r*) + export_code blexer_simp blexer lexer bders bders_simp in Scala module_name VerifiedLexers