Theory ArrayHashMap_Impl

theory ArrayHashMap_Impl
imports HashCode Code_Target_ICF ListGA ListMapImpl Array_Iterator
(*  Title:       Isabelle Collections Library
    Author:      Andreas Lochbihler <andreas dot lochbihler at kit.edu>
    Maintainer:  Andreas Lochbihler <andreas dot lochbihler at kit.edu>
*)
section ‹\isaheader{Array-based hash map implementation}›
theory ArrayHashMap_Impl imports 
  "../../Lib/HashCode"
  "../../Lib/Code_Target_ICF"
  "../../Lib/Diff_Array"
  "../gen_algo/ListGA"
  ListMapImpl
  "../../Iterator/Array_Iterator"
begin

text ‹Misc.›

setup Locale_Code.open_block
interpretation a_idx_it: 
  idx_iteratei_loc list_of_array "λ_. True" array_length array_get
  apply unfold_locales
  apply (case_tac [!] s) [2]
  apply auto
  done
setup Locale_Code.close_block

(*
lemma idx_iteratei_aux_array_get_Array_conv_nth:
  "idx_iteratei_aux array_get sz i (Array xs) c f σ = idx_iteratei_aux (!) sz i xs c f σ"
apply(induct get≡"(!) :: 'b list ⇒ nat ⇒ 'b" sz i xs c f σ rule: idx_iteratei_aux.induct)
apply(subst (1 2) idx_iteratei_aux.simps)
apply simp
done

lemma idx_iteratei_array_get_Array_conv_nth:
  "idx_iteratei array_get array_length (Array xs) = idx_iteratei nth length xs"
by(simp add: idx_iteratei_def fun_eq_iff idx_iteratei_aux_array_get_Array_conv_nth)

lemma idx_iteratei_aux_nth_conv_foldli_drop:
  fixes xs :: "'b list"
  assumes "i ≤ length xs"
  shows "idx_iteratei_aux (!) (length xs) i xs c f σ = foldli (drop (length xs - i) xs) c f σ"
using assms
proof(induct get≡"(!) :: 'b list ⇒ nat ⇒ 'b" sz≡"length xs" i xs c f σ rule: idx_iteratei_aux.induct)
  case (1 i l c f σ)
  show ?case
  proof(cases "i = 0 ∨ ¬ c σ")
    case True thus ?thesis
      by(subst idx_iteratei_aux.simps)(auto)
  next
    case False
    hence i: "i > 0" and c: "c σ" by auto
    hence "idx_iteratei_aux (!) (length l) i l c f σ = idx_iteratei_aux (!) (length l) (i - 1) l c f (f (l ! (length l - i)) σ)"
      by(subst idx_iteratei_aux.simps) simp
    also have "… = foldli (drop (length l - (i - 1)) l) c f (f (l ! (length l - i)) σ)"
      using `i ≤ length l` i c by -(rule 1, auto)
    also from `i ≤ length l` i
    have "drop (length l - i) l = (l ! (length l - i)) # drop (length l - (i - 1)) l"
      by(subst Cons_nth_drop_Suc[symmetric])(simp_all, metis Suc_eq_plus1_left add_diff_assoc)
    hence "foldli (drop (length l - (i - 1)) l) c f (f (l ! (length l - i)) σ) = foldli (drop (length l - i) l) c f σ"
      using c by simp
    finally show ?thesis .
  qed
qed

lemma idx_iteratei_nth_length_conv_foldli: "idx_iteratei nth length = foldli"
by(rule ext)+(simp add: idx_iteratei_def idx_iteratei_aux_nth_conv_foldli_drop)
*)

subsection ‹Type definition and primitive operations›

definition load_factor :: nat ― ‹in percent›
  where "load_factor = 75"

text ‹
  We do not use @{typ "('k, 'v) assoc_list"} for the buckets but plain lists of key-value pairs.
  This speeds up rehashing because we then do not have to go through the abstract operations.
›

datatype ('key, 'val) hashmap =
  HashMap "('key × 'val) list array" "nat"

subsection ‹Operations›

definition new_hashmap_with :: "nat ⇒ ('key :: hashable, 'val) hashmap"
where "⋀size. new_hashmap_with size = HashMap (new_array [] size) 0"

definition ahm_empty :: "unit ⇒ ('key :: hashable, 'val) hashmap"
where "ahm_empty ≡ λ_. new_hashmap_with (def_hashmap_size TYPE('key))"

definition bucket_ok :: "nat ⇒ nat ⇒ (('key :: hashable) × 'val) list ⇒ bool"
where "bucket_ok len h kvs = (∀k ∈ fst ` set kvs. bounded_hashcode_nat len k = h)"

definition ahm_invar_aux :: "nat ⇒ (('key :: hashable) × 'val) list array ⇒ bool"
where
  "ahm_invar_aux n a ⟷
  (∀h. h < array_length a ⟶ bucket_ok (array_length a) h (array_get a h) ∧ distinct (map fst (array_get a h))) ∧
  array_foldl (λ_ n kvs. n + size kvs) 0 a = n ∧
  array_length a > 1"


primrec ahm_invar :: "('key :: hashable, 'val) hashmap ⇒ bool"
where "ahm_invar (HashMap a n) = ahm_invar_aux n a"

definition ahm_α_aux :: "(('key :: hashable) × 'val) list array ⇒ 'key ⇒ 'val option"
where [simp]: "ahm_α_aux a k = map_of (array_get a (bounded_hashcode_nat (array_length a) k)) k"

primrec ahm_α :: "('key :: hashable, 'val) hashmap ⇒ 'key ⇒ 'val option"
where
  "ahm_α (HashMap a _) = ahm_α_aux a"

definition ahm_lookup :: "'key ⇒ ('key :: hashable, 'val) hashmap ⇒ 'val option"
where "ahm_lookup k hm  = ahm_α hm k"

primrec ahm_iteratei_aux :: "((('key :: hashable) × 'val) list array) ⇒ ('key × 'val, 'σ) set_iterator"
where "ahm_iteratei_aux (Array xs) c f = foldli (concat xs) c f"

primrec ahm_iteratei :: "(('key :: hashable, 'val) hashmap) ⇒ (('key × 'val), 'σ) set_iterator"
where
  "ahm_iteratei (HashMap a n) = ahm_iteratei_aux a"

definition ahm_rehash_aux' :: "nat ⇒ 'key × 'val ⇒ (('key :: hashable) × 'val) list array ⇒ ('key × 'val) list array"
where
  "ahm_rehash_aux' n kv a =
   (let h = bounded_hashcode_nat n (fst kv)
    in array_set a h (kv # array_get a h))"

definition ahm_rehash_aux :: "(('key :: hashable) × 'val) list array ⇒ nat ⇒ ('key × 'val) list array"
where
  "ahm_rehash_aux a sz = ahm_iteratei_aux a (λx. True) (ahm_rehash_aux' sz) (new_array [] sz)"

primrec ahm_rehash :: "('key :: hashable, 'val) hashmap ⇒ nat ⇒ ('key, 'val) hashmap"
where "ahm_rehash (HashMap a n) sz = HashMap (ahm_rehash_aux a sz) n"

primrec hm_grow :: "('key :: hashable, 'val) hashmap ⇒ nat"
where "hm_grow (HashMap a n) = 2 * array_length a + 3"

primrec ahm_filled :: "('key :: hashable, 'val) hashmap ⇒ bool"
where "ahm_filled (HashMap a n) = (array_length a * load_factor ≤ n * 100)"

primrec ahm_update_aux :: "('key :: hashable, 'val) hashmap ⇒ 'key ⇒ 'val ⇒ ('key, 'val) hashmap"
where
  "ahm_update_aux (HashMap a n) k v = 
  (let h = bounded_hashcode_nat (array_length a) k;
       m = array_get a h;
       insert = map_of m k = None
   in HashMap (array_set a h (AList.update k v m)) (if insert then n + 1 else n))"

definition ahm_update :: "'key ⇒ 'val ⇒ ('key :: hashable, 'val) hashmap ⇒ ('key, 'val) hashmap"
where
  "ahm_update k v hm = 
   (let hm' = ahm_update_aux hm k v
    in (if ahm_filled hm' then ahm_rehash hm' (hm_grow hm') else hm'))"

primrec ahm_delete :: "'key ⇒ ('key :: hashable, 'val) hashmap ⇒ ('key, 'val) hashmap"
where
  "ahm_delete k (HashMap a n) =
  (let h = bounded_hashcode_nat (array_length a) k;
       m = array_get a h;
       deleted = (map_of m k ≠ None)
   in HashMap (array_set a h (AList.delete k m)) (if deleted then n - 1 else n))"


lemma hm_grow_gt_1 [iff]:
  "Suc 0 < hm_grow hm"
by(cases hm)(simp)

lemma bucket_ok_Nil [simp]: "bucket_ok len h [] = True"
by(simp add: bucket_ok_def)

lemma bucket_okD:
  "⟦ bucket_ok len h xs; (k, v) ∈ set xs ⟧
  ⟹ bounded_hashcode_nat len k = h"
by(auto simp add: bucket_ok_def)

lemma bucket_okI:
  "(⋀k. k ∈ fst ` set kvs ⟹ bounded_hashcode_nat len k = h) ⟹ bucket_ok len h kvs"
by(simp add: bucket_ok_def)


subsection ‹@{term ahm_invar}›

lemma ahm_invar_auxE:
  assumes "ahm_invar_aux n a"
  obtains "∀h. h < array_length a ⟶ bucket_ok (array_length a) h (array_get a h) ∧ distinct (map fst (array_get a h))"
  and "n = array_foldl (λ_ n kvs. n + length kvs) 0 a" and "array_length a > 1"
using assms unfolding ahm_invar_aux_def by blast

lemma ahm_invar_auxI:
  "⟦ ⋀h. h < array_length a ⟹ bucket_ok (array_length a) h (array_get a h);
     ⋀h. h < array_length a ⟹ distinct (map fst (array_get a h));
     n = array_foldl (λ_ n kvs. n + length kvs) 0 a; array_length a > 1 ⟧
  ⟹ ahm_invar_aux n a"
unfolding ahm_invar_aux_def by blast

lemma ahm_invar_distinct_fst_concatD:
  assumes inv: "ahm_invar_aux n (Array xs)"
  shows "distinct (map fst (concat xs))"
proof -
  { fix h
    assume "h < length xs"
    with inv have "bucket_ok (length xs) h (xs ! h)" "distinct (map fst (xs ! h))"
      by(simp_all add: ahm_invar_aux_def) }
  note no_junk = this

  show ?thesis unfolding map_concat
  proof(rule distinct_concat')
    have "distinct [x←xs . x ≠ []]" unfolding distinct_conv_nth
    proof(intro allI ballI impI)
      fix i j
      assume "i < length [x←xs . x ≠ []]" "j < length [x←xs . x ≠ []]" "i ≠ j"
      from filter_nth_ex_nth[OF ‹i < length [x←xs . x ≠ []]›]
      obtain i' where "i' ≥ i" "i' < length xs" and ith: "[x←xs . x ≠ []] ! i = xs ! i'" 
        and eqi: "[x←take i' xs . x ≠ []] = take i [x←xs . x ≠ []]" by blast
      from filter_nth_ex_nth[OF ‹j < length [x←xs . x ≠ []]›]
      obtain j' where "j' ≥ j" "j' < length xs" and jth: "[x←xs . x ≠ []] ! j = xs ! j'"
        and eqj: "[x←take j' xs . x ≠ []] = take j [x←xs . x ≠ []]" by blast
      show "[x←xs . x ≠ []] ! i ≠ [x←xs . x ≠ []] ! j"
      proof
        assume "[x←xs . x ≠ []] ! i = [x←xs . x ≠ []] ! j"
        hence eq: "xs ! i' = xs ! j'" using ith jth by simp
        from ‹i < length [x←xs . x ≠ []]›
        have "[x←xs . x ≠ []] ! i ∈ set [x←xs . x ≠ []]" by(rule nth_mem)
        with ith have "xs ! i' ≠ []" by simp
        then obtain kv where "kv ∈ set (xs ! i')" by(fastforce simp add: neq_Nil_conv)
        with no_junk[OF ‹i' < length xs›] have "bounded_hashcode_nat (length xs) (fst kv) = i'"
          by(simp add: bucket_ok_def)
        moreover from eq ‹kv ∈ set (xs ! i')› have "kv ∈ set (xs ! j')" by simp
        with no_junk[OF ‹j' < length xs›] have "bounded_hashcode_nat (length xs) (fst kv) = j'"
          by(simp add: bucket_ok_def)
        ultimately have [simp]: "i' = j'" by simp
        from ‹i < length [x←xs . x ≠ []]› have "i = length (take i [x←xs . x ≠ []])" by simp
        also from eqi eqj have "take i [x←xs . x ≠ []] = take j [x←xs . x ≠ []]" by simp
        finally show False using ‹i ≠ j› ‹j < length [x←xs . x ≠ []]› by simp
      qed
    qed
    moreover have "inj_on (map fst) {x ∈ set xs. x ≠ []}"
    proof(rule inj_onI)
      fix x y
      assume "x ∈ {x ∈ set xs. x ≠ []}" "y ∈ {x ∈ set xs. x ≠ []}" "map fst x = map fst y"
      hence "x ∈ set xs" "y ∈ set xs" "x ≠ []" "y ≠ []" by auto
      from ‹x ∈ set xs› obtain i where "xs ! i = x" "i < length xs" unfolding set_conv_nth by fastforce
      from ‹y ∈ set xs› obtain j where "xs ! j = y" "j < length xs" unfolding set_conv_nth by fastforce
      from ‹x ≠ []› obtain k v x' where "x = (k, v) # x'" by(cases x) auto
      with no_junk[OF ‹i < length xs›] ‹xs ! i = x›
      have "bounded_hashcode_nat (length xs) k = i" by(auto simp add: bucket_ok_def)
      moreover from ‹map fst x = map fst y› ‹x = (k, v) # x'› obtain v' where "(k, v') ∈ set y" by fastforce
      with no_junk[OF ‹j < length xs›] ‹xs ! j = y›
      have "bounded_hashcode_nat (length xs) k = j" by(auto simp add: bucket_ok_def)
      ultimately have "i = j" by simp
      with ‹xs ! i = x› ‹xs ! j = y› show "x = y" by simp
    qed
    ultimately show "distinct [ys←map (map fst) xs . ys ≠ []]"
      by(simp add: filter_map o_def distinct_map)
  next
    fix ys
    assume "ys ∈ set (map (map fst) xs)"
    thus "distinct ys" by(clarsimp simp add: set_conv_nth)(rule no_junk)
  next
    fix ys zs
    assume "ys ∈ set (map (map fst) xs)" "zs ∈ set (map (map fst) xs)" "ys ≠ zs"
    then obtain ys' zs' where [simp]: "ys = map fst ys'" "zs = map fst zs'" 
      and "ys' ∈ set xs" "zs' ∈ set xs" by auto
    have "fst ` set ys' ∩ fst ` set zs' = {}"
    proof(rule equals0I)
      fix k
      assume "k ∈ fst ` set ys' ∩ fst ` set zs'"
      then obtain v v' where "(k, v) ∈ set ys'" "(k, v') ∈ set zs'" by(auto)
      from ‹ys' ∈ set xs› obtain i where "xs ! i = ys'" "i < length xs" unfolding set_conv_nth by fastforce
      with ‹(k, v) ∈ set ys'› have "bounded_hashcode_nat (length xs) k = i" by(auto dest: no_junk bucket_okD)
      moreover
      from ‹zs' ∈ set xs› obtain j where "xs ! j = zs'" "j < length xs" unfolding set_conv_nth by fastforce
      with ‹(k, v') ∈ set zs'› have "bounded_hashcode_nat (length xs) k = j" by(auto dest: no_junk bucket_okD)
      ultimately have "i = j" by simp
      with ‹xs ! i = ys'› ‹xs ! j = zs'› have "ys' = zs'" by simp
      with ‹ys ≠ zs› show False by simp
    qed
    thus "set ys ∩ set zs = {}" by simp
  qed
qed

subsection ‹@{term "ahm_α"}›

lemma finite_dom_ahm_α_aux:
  assumes "ahm_invar_aux n a"
  shows "finite (dom (ahm_α_aux a))"
proof -
  have "dom (ahm_α_aux a) ⊆ (⋃h ∈ range (bounded_hashcode_nat (array_length a) :: 'a ⇒ nat). dom (map_of (array_get a h)))"
    by(force simp add: dom_map_of_conv_image_fst ahm_α_aux_def dest: map_of_SomeD)
  moreover have "finite …"
  proof(rule finite_UN_I)
    from ‹ahm_invar_aux n a› have "array_length a > 1" by(simp add: ahm_invar_aux_def)
    hence "range (bounded_hashcode_nat (array_length a) :: 'a ⇒ nat) ⊆ {0..<array_length a}"
      by(auto simp add: bounded_hashcode_nat_bounds)
    thus "finite (range (bounded_hashcode_nat (array_length a) :: 'a ⇒ nat))"
      by(rule finite_subset) simp
  qed(rule finite_dom_map_of)
  ultimately show ?thesis by(rule finite_subset)
qed

lemma ahm_α_aux_conv_map_of_concat:
  assumes inv: "ahm_invar_aux n (Array xs)"
  shows "ahm_α_aux (Array xs) = map_of (concat xs)"
proof
  fix k
  show "ahm_α_aux (Array xs) k = map_of (concat xs) k"
  proof(cases "map_of (concat xs) k")
    case None
    hence "k ∉ fst ` set (concat xs)" by(simp add: map_of_eq_None_iff)
    hence "k ∉ fst ` set (xs ! bounded_hashcode_nat (length xs) k)"
    proof(rule contrapos_nn)
      assume "k ∈ fst ` set (xs ! bounded_hashcode_nat (length xs) k)"
      then obtain v where "(k, v) ∈ set (xs ! bounded_hashcode_nat (length xs) k)" by auto
      moreover from inv have "bounded_hashcode_nat (length xs) k < length xs"
        by(simp add: bounded_hashcode_nat_bounds ahm_invar_aux_def)
      ultimately show "k ∈ fst ` set (concat xs)"
        by(force intro: rev_image_eqI)
    qed
    thus ?thesis unfolding None by(simp add: map_of_eq_None_iff)
  next
    case (Some v)
    hence "(k, v) ∈ set (concat xs)" by(rule map_of_SomeD)
    then obtain ys where "ys ∈ set xs" "(k, v) ∈ set ys"
      unfolding set_concat by blast
    from ‹ys ∈ set xs› obtain i j where "i < length xs" "xs ! i = ys"
      unfolding set_conv_nth by auto
    with inv ‹(k, v) ∈ set ys›
    show ?thesis unfolding Some
      by(force dest: bucket_okD simp add: ahm_invar_aux_def)
  qed
qed

lemma ahm_invar_aux_card_dom_ahm_α_auxD:
  assumes inv: "ahm_invar_aux n a"
  shows "card (dom (ahm_α_aux a)) = n"
proof(cases a)
  case [simp]: (Array xs)
  from inv have "card (dom (ahm_α_aux (Array xs))) = card (dom (map_of (concat xs)))"
    by(simp add: ahm_α_aux_conv_map_of_concat)
  also from inv have "distinct (map fst (concat xs))"
    by(simp add: ahm_invar_distinct_fst_concatD)
  hence "card (dom (map_of (concat xs))) = length (concat xs)"
    by(rule card_dom_map_of)
  also have "length (concat xs) = foldl (+) 0 (map length xs)"
    by (simp add: length_concat foldl_conv_fold add.commute fold_plus_sum_list_rev)
  also from inv
  have "… = n" unfolding foldl_map by(simp add: ahm_invar_aux_def array_foldl_foldl)
  finally show ?thesis by(simp)
qed

lemma finite_dom_ahm_α:
  "ahm_invar hm ⟹ finite (dom (ahm_α hm))"
by(cases hm)(auto intro: finite_dom_ahm_α_aux)

lemma finite_map_ahm_α_aux:
  "finite_map ahm_α_aux (ahm_invar_aux n)"
by(unfold_locales)(rule finite_dom_ahm_α_aux)

lemma finite_map_ahm_α:
  "finite_map ahm_α ahm_invar"
by(unfold_locales)(rule finite_dom_ahm_α)

subsection ‹@{term ahm_empty}›

lemma ahm_invar_aux_new_array:
  assumes "n > 1"
  shows "ahm_invar_aux 0 (new_array [] n)"
proof -
  have "foldl (λb (k, v). b + length v) 0 (zip [0..<n] (replicate n [])) = 0"
    by(induct n)(simp_all add: replicate_Suc_conv_snoc del: replicate_Suc)
  with assms show ?thesis by(simp add: ahm_invar_aux_def array_foldl_new_array)
qed

lemma ahm_invar_new_hashmap_with:
  "n > 1 ⟹ ahm_invar (new_hashmap_with n)"
by(auto simp add: ahm_invar_def new_hashmap_with_def intro: ahm_invar_aux_new_array)

lemma ahm_α_new_hashmap_with:
  "n > 1 ⟹ ahm_α (new_hashmap_with n) = Map.empty"
by(simp add: new_hashmap_with_def bounded_hashcode_nat_bounds fun_eq_iff)

lemma ahm_invar_ahm_empty [simp]: "ahm_invar (ahm_empty ())"
using def_hashmap_size[where ?'a = 'a]
by(auto intro: ahm_invar_new_hashmap_with simp add: ahm_empty_def)

lemma ahm_empty_correct [simp]: "ahm_α (ahm_empty ()) = Map.empty"
using def_hashmap_size[where ?'a = 'a]
by(auto intro: ahm_α_new_hashmap_with simp add: ahm_empty_def)

lemma ahm_empty_impl: "map_empty ahm_α ahm_invar ahm_empty"
by(unfold_locales)(auto)

subsection ‹@{term "ahm_lookup"}›

lemma ahm_lookup_impl: "map_lookup ahm_α ahm_invar ahm_lookup"
by(unfold_locales)(simp add: ahm_lookup_def)

subsection ‹@{term "ahm_iteratei"}›

lemma ahm_iteratei_aux_impl:
  assumes invar_m: "ahm_invar_aux n m"
  shows "map_iterator (ahm_iteratei_aux m) (ahm_α_aux m)"
proof -
  obtain ms where m_eq[simp]: "m = Array ms" by (cases m)

  from ahm_invar_distinct_fst_concatD[of n ms] invar_m
  have dist: "distinct (map fst (concat ms))" by simp

  show "map_iterator (ahm_iteratei_aux m) (ahm_α_aux m)" 
    using  set_iterator_foldli_correct[of "concat ms"] dist
    by (simp add: ahm_α_aux_conv_map_of_concat[OF invar_m[unfolded m_eq]]
                  ahm_iteratei_aux_def map_to_set_map_of[OF dist] distinct_map)
qed 

lemma ahm_iteratei_correct:
  assumes invar_hm: "ahm_invar hm"
  shows "map_iterator (ahm_iteratei hm) (ahm_α hm)"
proof -
  obtain A n where hm_eq [simp]: "hm = HashMap A n" by(cases hm)

  from ahm_iteratei_aux_impl[of n A] invar_hm
    show map_it: "map_iterator (ahm_iteratei hm) (ahm_α hm)" by simp 
qed

lemma ahm_iteratei_aux_code [code]:
  "ahm_iteratei_aux a c f σ = a_idx_it.idx_iteratei a c (λx. foldli x c f) σ"
proof(cases a)
  case [simp]: (Array xs)

  have "ahm_iteratei_aux a c f σ = foldli (concat xs) c f σ" by simp
  also have "… = foldli xs c (λx. foldli x c f) σ" by (simp add: foldli_concat)
  thm a_idx_it.idx_iteratei_correct
  also have "… = a_idx_it.idx_iteratei a c (λx. foldli x c f) σ"
    by (simp add: a_idx_it.idx_iteratei_correct)
  finally show ?thesis .
qed
subsection ‹@{term "ahm_rehash"}›

lemma array_length_ahm_rehash_aux':
  "array_length (ahm_rehash_aux' n kv a) = array_length a"
by(simp add: ahm_rehash_aux'_def Let_def)

lemma ahm_rehash_aux'_preserves_ahm_invar_aux:
  assumes inv: "ahm_invar_aux n a"
  and fresh: "k ∉ fst ` set (array_get a (bounded_hashcode_nat (array_length a) k))"
  shows "ahm_invar_aux (Suc n) (ahm_rehash_aux' (array_length a) (k, v) a)"
  (is "ahm_invar_aux _ ?a")
proof(rule ahm_invar_auxI)
  fix h
  assume "h < array_length ?a"
  hence hlen: "h < array_length a" by(simp add: array_length_ahm_rehash_aux')
  with inv have bucket: "bucket_ok (array_length a) h (array_get a h)"
    and dist: "distinct (map fst (array_get a h))"
    by(auto elim: ahm_invar_auxE)
  let ?h = "bounded_hashcode_nat (array_length a) k"
  from hlen bucket show "bucket_ok (array_length ?a) h (array_get ?a h)"
    by(cases "h = ?h")(auto simp add: ahm_rehash_aux'_def Let_def array_length_ahm_rehash_aux' array_get_array_set_other dest: bucket_okD intro!: bucket_okI)
  from dist hlen fresh
  show "distinct (map fst (array_get ?a h))"
    by(cases "h = ?h")(auto simp add: ahm_rehash_aux'_def Let_def array_get_array_set_other)
next
  let ?f = "λn kvs. n + length kvs"
  { fix n :: nat and xs :: "('a × 'b) list list"
    have "foldl ?f n xs = n + foldl ?f 0 xs"
      by(induct xs arbitrary:  rule: rev_induct) simp_all }
  note fold = this
  let ?h = "bounded_hashcode_nat (array_length a) k"

  obtain xs where a [simp]: "a = Array xs" by(cases a)
  from inv have [simp]: "bounded_hashcode_nat (length xs) k < length xs"
    by(simp add: ahm_invar_aux_def bounded_hashcode_nat_bounds)
  have xs: "xs = take ?h xs @ (xs ! ?h) # drop (Suc ?h) xs" by(simp add: Cons_nth_drop_Suc)
  from inv have "n = array_foldl (λ_ n kvs. n + length kvs) 0 a"
    by(auto elim: ahm_invar_auxE)
  hence "n = foldl ?f 0 (take ?h xs) + length (xs ! ?h) + foldl ?f 0 (drop (Suc ?h) xs)"
    by(simp add: array_foldl_foldl)(subst xs, simp, subst (1 2 3 4) fold, simp)
  thus "Suc n = array_foldl (λ_ n kvs. n + length kvs) 0 ?a"
    by(simp add: ahm_rehash_aux'_def Let_def array_foldl_foldl foldl_list_update)(subst (1 2 3 4) fold, simp)
next
  from inv have "1 < array_length a" by(auto elim: ahm_invar_auxE)
  thus "1 < array_length ?a" by(simp add: array_length_ahm_rehash_aux')
qed

declare [[coercion_enabled = false]]

lemma ahm_rehash_aux_correct:
  fixes a :: "(('key :: hashable) × 'val) list array"
  assumes inv: "ahm_invar_aux n a"
  and "sz > 1"
  shows "ahm_invar_aux n (ahm_rehash_aux a sz)" (is "?thesis1")
  and "ahm_α_aux (ahm_rehash_aux a sz) = ahm_α_aux a" (is "?thesis2")
proof -
  (*interpret ahm: map_iterator "ahm_α_aux" "ahm_invar_aux n" "ahm_iteratei_aux"
    by(rule ahm_iteratei_aux_impl)*)
  let ?a = "ahm_rehash_aux a sz"
  let ?I = "λit a'. ahm_invar_aux (n - card it) a' ∧ array_length a' = sz ∧ (∀k. if k ∈ it then ahm_α_aux a' k = None else ahm_α_aux a' k = ahm_α_aux a k)"
  have "?I {} ?a ∨ (∃it⊆dom (ahm_α_aux a). it ≠ {} ∧ ¬ True ∧ ?I it ?a)"
    unfolding ahm_rehash_aux_def

  proof (rule map_iterator_rule_P[OF ahm_iteratei_aux_impl[OF inv], where
      c = "λ_. True" and f="ahm_rehash_aux' sz" and ?σ0.0 = "new_array [] sz"
      and I="?I"]
    )

    from inv have "card (dom (ahm_α_aux a)) = n" by(rule ahm_invar_aux_card_dom_ahm_α_auxD)
    moreover from ‹1 < sz› have "ahm_invar_aux 0 (new_array ([] :: ('key × 'val) list) sz)"
      by(rule ahm_invar_aux_new_array)
    moreover {
      fix k
      assume "k ∉ dom (ahm_α_aux a)"
      hence "ahm_α_aux a k = None" by auto
      moreover have "bounded_hashcode_nat sz k < sz" using ‹1 < sz›
        by(simp add: bounded_hashcode_nat_bounds)
      ultimately have "ahm_α_aux (new_array [] sz) k = ahm_α_aux a k" by simp }
    ultimately show "?I (dom (ahm_α_aux a)) (new_array [] sz)"
      by(auto simp add: bounded_hashcode_nat_bounds[OF ‹1 < sz›])
  next
    fix k :: 'key
      and v :: 'val
      and it a'
    assume "k ∈ it" "ahm_α_aux a k = Some v" 
      and it_sub: "it ⊆ dom (ahm_α_aux a)"
      and I: "?I it a'"
    from I have inv': "ahm_invar_aux (n - card it) a'" 
      and a'_eq_a: "⋀k. k ∉ it ⟹ ahm_α_aux a' k = ahm_α_aux a k" 
      and a'_None: "⋀k. k ∈ it ⟹ ahm_α_aux a' k = None"
      and [simp]: "sz = array_length a'" by(auto split: if_split_asm)
    from it_sub finite_dom_ahm_α_aux[OF inv] have "finite it" by(rule finite_subset)
    moreover with ‹k ∈ it› have "card it > 0" by(auto simp add: card_gt_0_iff)
    moreover from finite_dom_ahm_α_aux[OF inv] it_sub
    have "card it ≤ card (dom (ahm_α_aux a))" by(rule card_mono)
    moreover have "… = n" using inv
      by(simp add: ahm_invar_aux_card_dom_ahm_α_auxD)
    ultimately have "n - card (it - {k}) = (n - card it) + 1" using ‹k ∈ it› by auto
    moreover from ‹k ∈ it› have "ahm_α_aux a' k = None" by(rule a'_None)
    hence "k ∉ fst ` set (array_get a' (bounded_hashcode_nat (array_length a') k))"
      by(simp add: map_of_eq_None_iff)
    ultimately have "ahm_invar_aux (n - card (it - {k})) (ahm_rehash_aux' sz (k, v) a')"
      using inv' by(auto intro: ahm_rehash_aux'_preserves_ahm_invar_aux)
    moreover have "array_length (ahm_rehash_aux' sz (k, v) a') = sz"
      by(simp add: array_length_ahm_rehash_aux')
    moreover {
      fix k'
      assume "k' ∈ it - {k}"
      with bounded_hashcode_nat_bounds[OF ‹1 < sz›, of k'] a'_None[of k']
      have "ahm_α_aux (ahm_rehash_aux' sz (k, v) a') k' = None"
        by(cases "bounded_hashcode_nat sz k = bounded_hashcode_nat sz k'")(auto simp add: array_get_array_set_other ahm_rehash_aux'_def Let_def)
    } moreover {
      fix k'
      assume "k' ∉ it - {k}"
      with bounded_hashcode_nat_bounds[OF ‹1 < sz›, of k'] bounded_hashcode_nat_bounds[OF ‹1 < sz›, of k] a'_eq_a[of k'] ‹k ∈ it›
      have "ahm_α_aux (ahm_rehash_aux' sz (k, v) a') k' = ahm_α_aux a k'"
        unfolding ahm_rehash_aux'_def Let_def using ‹ahm_α_aux a k = Some v›
        by(cases "bounded_hashcode_nat sz k = bounded_hashcode_nat sz k'")(case_tac [!] "k' = k", simp_all add: array_get_array_set_other) }
    ultimately show "?I (it - {k}) (ahm_rehash_aux' sz (k, v) a')" by simp
  qed auto
  thus ?thesis1 ?thesis2 unfolding ahm_rehash_aux_def
    by(auto intro: ext)
qed

lemma ahm_rehash_correct:
  fixes hm :: "('key :: hashable, 'val) hashmap"
  assumes inv: "ahm_invar hm"
  and "sz > 1"
  shows "ahm_invar (ahm_rehash hm sz)" "ahm_α (ahm_rehash hm sz) = ahm_α hm"
using assms
by -(case_tac [!] hm, auto intro: ahm_rehash_aux_correct)

subsection ‹@{term ahm_update}›

lemma ahm_update_aux_correct:
  assumes inv: "ahm_invar hm"
  shows "ahm_invar (ahm_update_aux hm k v)" (is ?thesis1)
  and "ahm_α (ahm_update_aux hm k v) = (ahm_α hm)(k ↦ v)" (is ?thesis2)
proof -
  obtain a n where [simp]: "hm = HashMap a n" by(cases hm)

  let ?h = "bounded_hashcode_nat (array_length a) k"
  let ?a' = "array_set a ?h (AList.update k v (array_get a ?h))"
  let ?n' = "if map_of (array_get a ?h) k = None then n + 1 else n"

  have "ahm_invar (HashMap ?a' ?n')" unfolding ahm_invar.simps
  proof(rule ahm_invar_auxI)
    fix h
    assume "h < array_length ?a'"
    hence "h < array_length a" by simp
    with inv have "bucket_ok (array_length a) h (array_get a h)"
      by(auto elim: ahm_invar_auxE)
    thus "bucket_ok (array_length ?a') h (array_get ?a' h)"
      using ‹h < array_length a›
      apply(cases "h = bounded_hashcode_nat (array_length a) k")
      apply(fastforce intro!: bucket_okI simp add: dom_update array_get_array_set_other dest: bucket_okD del: imageE elim: imageE)+
      done
    from ‹h < array_length a› inv have "distinct (map fst (array_get a h))"
      by(auto elim: ahm_invar_auxE)
    with ‹h < array_length a›
    show "distinct (map fst (array_get ?a' h))"
      by(cases "h = bounded_hashcode_nat (array_length a) k")(auto simp add: array_get_array_set_other intro: distinct_update)
  next
    obtain xs where a [simp]: "a = Array xs" by(cases a)

    let ?f = "λn kvs. n + length kvs"
    { fix n :: nat and xs :: "('a × 'b) list list"
      have "foldl ?f n xs = n + foldl ?f 0 xs"
        by(induct xs arbitrary:  rule: rev_induct) simp_all }
    note fold = this

    from inv have [simp]: "bounded_hashcode_nat (length xs) k < length xs"
      by(simp add: ahm_invar_aux_def bounded_hashcode_nat_bounds)
    have xs: "xs = take ?h xs @ (xs ! ?h) # drop (Suc ?h) xs" by(simp add: Cons_nth_drop_Suc)
    from inv have "n = array_foldl (λ_ n kvs. n + length kvs) 0 a"
      by(auto elim: ahm_invar_auxE)
    hence "n = foldl ?f 0 (take ?h xs) + length (xs ! ?h) + foldl ?f 0 (drop (Suc ?h) xs)"
      by(simp add: array_foldl_foldl)(subst xs, simp, subst (1 2 3 4) fold, simp)
    thus "?n' = array_foldl (λ_ n kvs. n + length kvs) 0 ?a'"
      apply(simp add: ahm_rehash_aux'_def Let_def array_foldl_foldl foldl_list_update map_of_eq_None_iff)
      apply(subst (1 2 3 4 5 6 7 8) fold)
      apply(simp add: length_update)
      done
  next
    from inv have "1 < array_length a" by(auto elim: ahm_invar_auxE)
    thus "1 < array_length ?a'" by simp
  qed
  moreover have "ahm_α (ahm_update_aux hm k v) = ahm_α hm(k ↦ v)"
  proof
    fix k'
    from inv have "1 < array_length a" by(auto elim: ahm_invar_auxE)
    with bounded_hashcode_nat_bounds[OF this, of k]
    show "ahm_α (ahm_update_aux hm k v) k' = (ahm_α hm(k ↦ v)) k'"
      by(cases "bounded_hashcode_nat (array_length a) k = bounded_hashcode_nat (array_length a) k'")(auto simp add: Let_def update_conv array_get_array_set_other)
  qed
  ultimately show ?thesis1 ?thesis2 by(simp_all add: Let_def)
qed

lemma ahm_update_correct:
  assumes inv: "ahm_invar hm"
  shows "ahm_invar (ahm_update k v hm)"
  and "ahm_α (ahm_update k v hm) = (ahm_α hm)(k ↦ v)"
using assms
by(simp_all add: ahm_update_def Let_def ahm_rehash_correct ahm_update_aux_correct)

lemma ahm_update_impl:
  "map_update ahm_α ahm_invar ahm_update"
by(unfold_locales)(simp_all add: ahm_update_correct)

subsection ‹@{term "ahm_delete"}›

lemma ahm_delete_correct:
  assumes inv: "ahm_invar hm"
  shows "ahm_invar (ahm_delete k hm)" (is "?thesis1")
  and "ahm_α (ahm_delete k hm) = (ahm_α hm) |` (- {k})" (is "?thesis2")
proof -
  obtain a n where hm [simp]: "hm = HashMap a n" by(cases hm)

  let ?h = "bounded_hashcode_nat (array_length a) k"
  let ?a' = "array_set a ?h (AList.delete k (array_get a ?h))"
  let ?n' = "if map_of (array_get a (bounded_hashcode_nat (array_length a) k)) k = None then n else n - 1"
  
  have "ahm_invar_aux ?n' ?a'"
  proof(rule ahm_invar_auxI)
    fix h
    assume "h < array_length ?a'"
    hence "h < array_length a" by simp
    with inv have "bucket_ok (array_length a) h (array_get a h)"
      and "1 < array_length a" 
      and "distinct (map fst (array_get a h))" by(auto elim: ahm_invar_auxE)
    thus "bucket_ok (array_length ?a') h (array_get ?a' h)"
      and "distinct (map fst (array_get ?a' h))"
      using bounded_hashcode_nat_bounds[of "array_length a" k] 
      by-(case_tac [!] "h = bounded_hashcode_nat (array_length a) k", auto simp add: array_get_array_set_other set_delete_conv intro!: bucket_okI dest: bucket_okD intro: distinct_delete)
  next
    obtain xs where a [simp]: "a = Array xs" by(cases a)

    let ?f = "λn kvs. n + length kvs"
    { fix n :: nat and xs :: "('a × 'b) list list"
      have "foldl ?f n xs = n + foldl ?f 0 xs"
        by(induct xs arbitrary:  rule: rev_induct) simp_all }
    note fold = this

    from inv have [simp]: "bounded_hashcode_nat (length xs) k < length xs"
      by(simp add: ahm_invar_aux_def bounded_hashcode_nat_bounds)
    from inv have "distinct (map fst (array_get a ?h))" by(auto elim: ahm_invar_auxE)
    moreover
    have xs: "xs = take ?h xs @ (xs ! ?h) # drop (Suc ?h) xs" by(simp add: Cons_nth_drop_Suc)
    from inv have "n = array_foldl (λ_ n kvs. n + length kvs) 0 a"
      by(auto elim: ahm_invar_auxE)
    hence "n = foldl ?f 0 (take ?h xs) + length (xs ! ?h) + foldl ?f 0 (drop (Suc ?h) xs)"
      by(simp add: array_foldl_foldl)(subst xs, simp, subst (1 2 3 4) fold, simp)
    ultimately show "?n' = array_foldl (λ_ n kvs. n + length kvs) 0 ?a'"
      apply(simp add: array_foldl_foldl foldl_list_update map_of_eq_None_iff)
      apply(subst (1 2 3 4 5 6 7 8) fold)
      apply(auto simp add: length_distinct in_set_conv_nth)
      done
  next
    from inv show "1 < array_length ?a'" by(auto elim: ahm_invar_auxE)
  qed
  thus "?thesis1" by(auto simp add: Let_def)

  have "ahm_α_aux ?a' = ahm_α_aux a |` (- {k})"
  proof
    fix k' :: 'a
    from inv have "bounded_hashcode_nat (array_length a) k < array_length a"
      by(auto elim: ahm_invar_auxE simp add: bounded_hashcode_nat_bounds)
    thus "ahm_α_aux ?a' k' = (ahm_α_aux a |` (- {k})) k'"
      by(cases "?h = bounded_hashcode_nat (array_length a) k'")(auto simp add: restrict_map_def array_get_array_set_other delete_conv)
  qed
  thus ?thesis2 by(simp add: Let_def)
qed

lemma ahm_delete_impl:
  "map_delete ahm_α ahm_invar ahm_delete"
by(unfold_locales)(blast intro: ahm_delete_correct)+

hide_const (open) HashMap ahm_empty bucket_ok ahm_invar ahm_α ahm_lookup
  ahm_iteratei ahm_rehash hm_grow ahm_filled ahm_update ahm_delete
hide_type (open) hashmap

end