diff -r b732997cfc11 -r 42d11e0a7a8b src/HOL/MicroJava/BV/Step.thy --- a/src/HOL/MicroJava/BV/Step.thy Mon Aug 14 14:57:29 2000 +0200 +++ b/src/HOL/MicroJava/BV/Step.thy Mon Aug 14 18:03:19 2000 +0200 @@ -10,7 +10,7 @@ theory Step = Convert : -text "Effect of instruction on the state type" +text "Effect of instruction on the state type:" consts step :: "instr \ jvm_prog \ state_type \ state_type option" @@ -39,7 +39,7 @@ "step (i,G,s) = None" -text "Conditions under which step is applicable" +text "Conditions under which step is applicable:" consts app :: "instr \ jvm_prog \ ty \ state_type \ bool" @@ -84,7 +84,7 @@ "app (i,G,rT,s) = False" -text {* \verb,p_count, of successor instructions *} +text {* program counter of successor instructions: *} consts succs :: "instr \ p_count \ p_count set" @@ -134,10 +134,8 @@ text {* \medskip -simp rules for @{term app} without patterns, better suited for proofs -\medskip +simp rules for \isa{app} without patterns, better suited for proofs: *} - lemma appStore[simp]: "app (Store idx, G, rT, s) = (\ ts ST LT. s = (ts#ST,LT) \ idx < length LT)" by (cases s, cases "2 < length (fst s)", auto dest: 1 2)