changeset 51094 | 84b03c49c223 |
parent 50138 | ca989d793b34 |
child 51143 | 0a2371e7ced3 |
--- a/src/HOL/ex/IArray_Examples.thy Wed Feb 13 13:38:52 2013 +0100 +++ b/src/HOL/ex/IArray_Examples.thy Wed Feb 13 13:38:52 2013 +0100 @@ -1,5 +1,5 @@ theory IArray_Examples -imports "~~/src/HOL/Library/IArray" +imports "~~/src/HOL/Library/IArray" "~~/src/HOL/Library/Efficient_Nat" begin lemma "IArray [True,False] !! 1 = False" @@ -24,3 +24,4 @@ by eval end +