thys/Lexer.thy
changeset 257 9deaff82e0c5
parent 256 146b4817aebd
child 261 247fc5dd4943
--- a/thys/Lexer.thy	Thu Jun 29 17:57:41 2017 +0100
+++ b/thys/Lexer.thy	Fri Jun 30 17:41:45 2017 +0100
@@ -1,6 +1,6 @@
    
 theory Lexer
-  imports Main
+  imports Main 
 begin
 
 
@@ -701,5 +701,4 @@
 using Posix1(1) Posix_determ lexer_correct_None lexer_correct_Some apply fastforce
 using Posix1(1) lexer_correct_None lexer_correct_Some by blast
 
-
 end
\ No newline at end of file