equal
deleted
inserted
replaced
2 ID: $Id$ |
2 ID: $Id$ |
3 Author: Gerwin Klein, Martin Strecker |
3 Author: Gerwin Klein, Martin Strecker |
4 Copyright 2001 Technische Universitaet Muenchen |
4 Copyright 2001 Technische Universitaet Muenchen |
5 *) |
5 *) |
6 |
6 |
7 header {* Exception handling in the JVM *} |
7 header {* \isaheader{Exception handling in the JVM} *} |
8 |
8 |
9 theory JVMExceptions = JVMInstructions: |
9 theory JVMExceptions = JVMInstructions: |
10 |
10 |
11 constdefs |
11 constdefs |
12 match_exception_entry :: "jvm_prog \<Rightarrow> cname \<Rightarrow> p_count \<Rightarrow> exception_entry \<Rightarrow> bool" |
12 match_exception_entry :: "jvm_prog \<Rightarrow> cname \<Rightarrow> p_count \<Rightarrow> exception_entry \<Rightarrow> bool" |