src/HOL/Imperative_HOL/ex/Subarray.thy
changeset 36098 53992c639da5
parent 30689 b14b2cc4e25e
child 37719 271ecd4fb9f9
equal deleted inserted replaced
36097:32383448c01b 36098:53992c639da5
       
     1 (*  Title:      HOL/Imperative_HOL/ex/Subarray.thy
       
     2     Author:     Lukas Bulwahn, TU Muenchen
       
     3 *)
       
     4 
       
     5 header {* Theorems about sub arrays *}
       
     6 
     1 theory Subarray
     7 theory Subarray
     2 imports Array Sublist
     8 imports Array Sublist
     3 begin
     9 begin
     4 
    10 
     5 definition subarray :: "nat \<Rightarrow> nat \<Rightarrow> ('a::heap) array \<Rightarrow> heap \<Rightarrow> 'a list"
    11 definition subarray :: "nat \<Rightarrow> nat \<Rightarrow> ('a::heap) array \<Rightarrow> heap \<Rightarrow> 'a list"