diff -r 5af61c89f51e -r 3ed514e2d93c thys3/src/BlexerSimp.thy --- a/thys3/src/BlexerSimp.thy Sun Jul 17 13:07:05 2022 +0100 +++ b/thys3/src/BlexerSimp.thy Sun Jul 17 20:09:38 2022 +0100 @@ -2,6 +2,15 @@ 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 = []"