diff -r a273bdac0934 -r 8b5f00202e1a src/HOL/MicroJava/BV/Effect.thy --- a/src/HOL/MicroJava/BV/Effect.thy Wed Oct 07 19:45:00 2015 +0200 +++ b/src/HOL/MicroJava/BV/Effect.thy Wed Oct 07 23:28:49 2015 +0200 @@ -3,7 +3,7 @@ Copyright 2000 Technische Universitaet Muenchen *) -section {* Effect of Instructions on the State Type *} +section \Effect of Instructions on the State Type\ theory Effect imports JVMType "../JVM/JVMExceptions" @@ -11,7 +11,7 @@ type_synonym succ_type = "(p_count \ state_type option) list" -text {* Program counter of successor instructions: *} +text \Program counter of successor instructions:\ primrec succs :: "instr \ p_count \ p_count list" where "succs (Load idx) pc = [pc+1]" | "succs (Store idx) pc = [pc+1]" @@ -226,10 +226,10 @@ lemmas [simp] = app_def xcpt_app_def -text {* +text \ \medskip simp rules for @{term app} -*} +\ lemma appNone[simp]: "app i G maxs rT pc et None = True" by simp