src/HOL/IMP/ASM.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58889 5b7a9633cfa8
equal deleted inserted replaced
58309:a09ec6daaa19 58310:91ea607a34d8
     3 theory ASM imports AExp begin
     3 theory ASM imports AExp begin
     4 
     4 
     5 subsection "Stack Machine"
     5 subsection "Stack Machine"
     6 
     6 
     7 text_raw{*\snip{ASMinstrdef}{0}{1}{% *}
     7 text_raw{*\snip{ASMinstrdef}{0}{1}{% *}
     8 datatype_new instr = LOADI val | LOAD vname | ADD
     8 datatype instr = LOADI val | LOAD vname | ADD
     9 text_raw{*}%endsnip*}
     9 text_raw{*}%endsnip*}
    10 
    10 
    11 text_raw{*\snip{ASMstackdef}{1}{2}{% *}
    11 text_raw{*\snip{ASMstackdef}{1}{2}{% *}
    12 type_synonym stack = "val list"
    12 type_synonym stack = "val list"
    13 text_raw{*}%endsnip*}
    13 text_raw{*}%endsnip*}