src/HOL/MicroJava/JVM/JVMExceptions.thy
changeset 58886 8a6cac7c7247
parent 39758 b8a53e3a0ee2
child 61361 8b5f00202e1a
equal deleted inserted replaced
58885:47fdd4f40d00 58886:8a6cac7c7247
     1 (*  Title:      HOL/MicroJava/JVM/JVMExceptions.thy
     1 (*  Title:      HOL/MicroJava/JVM/JVMExceptions.thy
     2     Author:     Gerwin Klein, Martin Strecker
     2     Author:     Gerwin Klein, Martin Strecker
     3     Copyright   2001 Technische Universitaet Muenchen
     3     Copyright   2001 Technische Universitaet Muenchen
     4 *)
     4 *)
     5 
     5 
     6 header {* \isaheader{Exception handling in the JVM} *}
     6 section {* Exception handling in the JVM *}
     7 
     7 
     8 theory JVMExceptions imports JVMInstructions begin
     8 theory JVMExceptions imports JVMInstructions begin
     9 
     9 
    10 definition match_exception_entry :: "jvm_prog \<Rightarrow> cname \<Rightarrow> p_count \<Rightarrow> exception_entry \<Rightarrow> bool" where
    10 definition match_exception_entry :: "jvm_prog \<Rightarrow> cname \<Rightarrow> p_count \<Rightarrow> exception_entry \<Rightarrow> bool" where
    11   "match_exception_entry G cn pc ee == 
    11   "match_exception_entry G cn pc ee ==