thys/Lexer.thy
changeset 257 9deaff82e0c5
parent 256 146b4817aebd
child 261 247fc5dd4943
equal deleted inserted replaced
256:146b4817aebd 257:9deaff82e0c5
     1    
     1    
     2 theory Lexer
     2 theory Lexer
     3   imports Main
     3   imports Main 
     4 begin
     4 begin
     5 
     5 
     6 
     6 
     7 section {* Sequential Composition of Languages *}
     7 section {* Sequential Composition of Languages *}
     8 
     8 
   699   shows "(lexer r s = Some v) \<longleftrightarrow> s \<in> r \<rightarrow> v"
   699   shows "(lexer r s = Some v) \<longleftrightarrow> s \<in> r \<rightarrow> v"
   700   and   "(lexer r s = None) \<longleftrightarrow> \<not>(\<exists>v. s \<in> r \<rightarrow> v)"
   700   and   "(lexer r s = None) \<longleftrightarrow> \<not>(\<exists>v. s \<in> r \<rightarrow> v)"
   701 using Posix1(1) Posix_determ lexer_correct_None lexer_correct_Some apply fastforce
   701 using Posix1(1) Posix_determ lexer_correct_None lexer_correct_Some apply fastforce
   702 using Posix1(1) lexer_correct_None lexer_correct_Some by blast
   702 using Posix1(1) lexer_correct_None lexer_correct_Some by blast
   703 
   703 
   704 
       
   705 end
   704 end