src/HOL/IMP/Compiler.thy
changeset 10343 24c87e1366d8
parent 10342 b124d59f7b61
child 10425 cab4acf9276d
equal deleted inserted replaced
10342:b124d59f7b61 10343:24c87e1366d8
       
     1 (*  Title:      HOL/IMP/Compiler.thy
       
     2     ID:         $Id$
       
     3     Author:     Tobias Nipkow, TUM
       
     4     Copyright   1996 TUM
       
     5 
       
     6 A simple compiler for a simplistic machine.
       
     7 *)
       
     8 
     1 theory Compiler = Natural:
     9 theory Compiler = Natural:
     2 
    10 
     3 datatype instr = ASIN loc aexp | JMPF bexp nat | JMPB nat
    11 datatype instr = ASIN loc aexp | JMPF bexp nat | JMPB nat
     4 
    12 
     5 consts  stepa1 :: "instr list => ((state*nat) * (state*nat))set"
    13 consts  stepa1 :: "instr list => ((state*nat) * (state*nat))set"