src/HOL/Library/Code_Index.thy
changeset 30663 0b6aff7451b2
parent 30245 e67f42ac1157
child 30926 3a30613aa469
equal deleted inserted replaced
30662:396be15b95d5 30663:0b6aff7451b2
     1 (* Author: Florian Haftmann, TU Muenchen *)
     1 (* Author: Florian Haftmann, TU Muenchen *)
     2 
     2 
     3 header {* Type of indices *}
     3 header {* Type of indices *}
     4 
     4 
     5 theory Code_Index
     5 theory Code_Index
     6 imports Plain "~~/src/HOL/Code_Eval" "~~/src/HOL/Presburger"
     6 imports Main
     7 begin
     7 begin
     8 
     8 
     9 text {*
     9 text {*
    10   Indices are isomorphic to HOL @{typ nat} but
    10   Indices are isomorphic to HOL @{typ nat} but
    11   mapped to target-language builtin integers.
    11   mapped to target-language builtin integers.