src/HOL/ex/IArray_Examples.thy
changeset 66453 cc19f7ca2ed6
parent 54459 f43ae1afd08a
child 69908 1bd74a0944b3
equal deleted inserted replaced
66452:450cefec7c11 66453:cc19f7ca2ed6
     1 theory IArray_Examples
     1 theory IArray_Examples
     2 imports "~~/src/HOL/Library/IArray" "~~/src/HOL/Library/Code_Target_Numeral"
     2 imports "HOL-Library.IArray" "HOL-Library.Code_Target_Numeral"
     3 begin
     3 begin
     4 
     4 
     5 lemma "IArray [True,False] !! 1 = False"
     5 lemma "IArray [True,False] !! 1 = False"
     6 by eval
     6 by eval
     7 
     7