thys/abacus.thy
changeset 63 35fe8fe12e65
parent 61 7edbd5657702
child 101 06db15939b7c
equal deleted inserted replaced
62:e33306b4c62e 63:35fe8fe12e65
     1 header {* 
     1 header {* 
     2  {\em abacus} a kind of register machine
     2  {\em abacus} a kind of register machine
     3 *}
     3 *}
     4 
     4 
     5 theory abacus
     5 theory abacus
     6 imports Main turing_hoare
     6 imports Main turing_basic
     7 begin
     7 begin
     8 
     8 
     9 text {*
     9 text {*
    10   {\em Abacus} instructions:
    10   {\em Abacus} instructions:
    11 *}
    11 *}