added paper
authorChristian Urban <christian.urban@kcl.ac.uk>
Sun, 17 Jul 2022 20:09:38 +0100
changeset 570 3ed514e2d93c
parent 569 5af61c89f51e
child 571 a76458dd9e4c
added paper
Literature/linear-lexer.pdf
thys3/src/BlexerSimp.thy
Binary file Literature/linear-lexer.pdf has changed
--- 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 \<Longrightarrow> P"
+  shows "~P \<Longrightarrow> ~Q"
+  using assms
+  apply(erule_tac contrapos_nn)
+  apply(simp)
+  done
+
 fun distinctWith :: "'a list \<Rightarrow> ('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a list"
   where
   "distinctWith [] eq acc = []"