diff -r a76458dd9e4c -r 344a834a093a thys3/src/BlexerSimp.thy --- a/thys3/src/BlexerSimp.thy Sun Jul 17 20:28:04 2022 +0100 +++ b/thys3/src/BlexerSimp.thy Sun Jul 17 20:28:46 2022 +0100 @@ -2,15 +2,6 @@ imports Blexer begin - -lemma test: - assumes "Q \ P" - shows "~P \ ~Q" - using assms - apply(erule_tac contrapos_nn) - apply(simp) - done - fun distinctWith :: "'a list \ ('a \ 'a \ bool) \ 'a set \ 'a list" where "distinctWith [] eq acc = []"