src/HOL/IMP/Compiler.thy
changeset 10425 cab4acf9276d
parent 10343 24c87e1366d8
child 11275 71498de45241
--- a/src/HOL/IMP/Compiler.thy	Thu Nov 09 21:38:30 2000 +0100
+++ b/src/HOL/IMP/Compiler.thy	Fri Nov 10 09:17:54 2000 +0100
@@ -27,7 +27,7 @@
 ASIN:  "P!n = ASIN x a ==> P |- <s,n> -1-> <s[x::= a s],Suc n>"
 JMPFT: "[| P!n = JMPF b i;  b s |] ==> P |- <s,n> -1-> <s,Suc n>"
 JMPFF: "[| P!n = JMPF b i; ~b s; m=n+i |] ==> P |- <s,n> -1-> <s,m>"
-JMPB:  "[| P!n = JMB i |] ==> P |- <s,n> -1-> <s,n-i>"
+JMPB:  "[| P!n = JMPB i |] ==> P |- <s,n> -1-> <s,n-i>"
 
 consts compile :: "com => instr list"
 primrec