added another definition snipped
authorkleing
Sun, 14 Apr 2013 21:54:45 +1000
changeset 51705 3d213f39d83c
parent 51704 0b0fc7dc4ce4
child 51706 0a4b4735d8bd
added another definition snipped
src/HOL/IMP/Comp_Rev.thy
--- a/src/HOL/IMP/Comp_Rev.thy	Fri Apr 12 17:56:51 2013 +0200
+++ b/src/HOL/IMP/Comp_Rev.thy	Sun Apr 14 21:54:45 2013 +1000
@@ -17,12 +17,14 @@
   "P \<turnstile> c \<rightarrow>^(Suc n) c'' = (\<exists>c'. (P \<turnstile> c \<rightarrow> c') \<and> P \<turnstile> c' \<rightarrow>^n c'')"
 
 text {* The possible successor PCs of an instruction at position @{term n} *}
+text_raw{*\snip{isuccsdef}{0}{1}{% *}
 definition
   "isuccs i n \<equiv> case i of 
      JMP j \<Rightarrow> {n + 1 + j}
    | JMPLESS j \<Rightarrow> {n + 1 + j, n + 1}
    | JMPGE j \<Rightarrow> {n + 1 + j, n + 1}
    | _ \<Rightarrow> {n +1}"
+text_raw{*}%endsnip*}
 
 text {* The possible successors PCs of an instruction list *}
 definition