src/HOL/IMP/ASM.thy
changeset 45266 13b5fb92b9f5
parent 45257 12063e071d92
child 45275 7f6c2db48b71
--- a/src/HOL/IMP/ASM.thy	Tue Oct 25 15:59:15 2011 +0200
+++ b/src/HOL/IMP/ASM.thy	Tue Oct 25 16:09:02 2011 +0200
@@ -1,8 +1,8 @@
-header "Arithmetic Stack Machine and Compilation"
+header "Stack Machine and Compilation"
 
 theory ASM imports AExp begin
 
-subsection "Arithmetic Stack Machine"
+subsection "Stack Machine"
 
 text_raw{*\begin{isaverbatimwrite}\newcommand{\ASMinstrdef}{% *}
 datatype instr = LOADI val | LOAD vname | ADD