From ce8f5c8f67e41a74bfdf8f6d664ff4e45e9de850 Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Thu, 7 Sep 2023 16:06:14 +0200
Subject: Regenerate the test files and fix a proof

---
 tests/coq/hashmap_on_disk/HashmapMain_Funs.v |  6 +-----
 tests/coq/hashmap_on_disk/Primitives.v       | 14 ++++++++++++++
 2 files changed, 15 insertions(+), 5 deletions(-)

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index 657d5590..a85adbf2 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -208,10 +208,6 @@ Definition hashmap_hash_map_insert_no_resize_fwd_back
       |})
 .
 
-(** [core::num::u32::{8}::MAX] *)
-Definition core_num_u32_max_body : result u32 := Return 4294967295%u32.
-Definition core_num_u32_max_c : u32 := core_num_u32_max_body%global.
-
 (** [hashmap_main::hashmap::HashMap::{0}::move_elements_from_list]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Fixpoint hashmap_hash_map_move_elements_from_list_loop_fwd_back
@@ -282,7 +278,7 @@ Definition hashmap_hash_map_try_resize_fwd_back
   (T : Type) (n : nat) (self : Hashmap_hash_map_t T) :
   result (Hashmap_hash_map_t T)
   :=
-  max_usize <- scalar_cast U32 Usize core_num_u32_max_c;
+  max_usize <- scalar_cast U32 Usize core_u32_max;
   let capacity := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
   n1 <- usize_div max_usize 2%usize;
   let (i, i0) := self.(Hashmap_hash_map_max_load_factor) in
diff --git a/tests/coq/hashmap_on_disk/Primitives.v b/tests/coq/hashmap_on_disk/Primitives.v
index 71a2d9c3..8d6c9c8d 100644
--- a/tests/coq/hashmap_on_disk/Primitives.v
+++ b/tests/coq/hashmap_on_disk/Primitives.v
@@ -394,6 +394,20 @@ Notation "x s< y" := (scalar_ltb x y)  (at level 80) : Primitives_scope.
 Notation "x s>= y" := (scalar_geb x y)  (at level 80) : Primitives_scope.
 Notation "x s> y" := (scalar_gtb x y)  (at level 80) : Primitives_scope.
 
+(** Constants *)
+Definition core_u8_max    := u8_max %u32.
+Definition core_u16_max   := u16_max %u32.
+Definition core_u32_max   := u32_max %u32.
+Definition core_u64_max   := u64_max %u64.
+Definition core_u128_max  := u64_max %u128.
+Axiom core_usize_max : usize. (** TODO *)
+Definition core_i8_max    := i8_max %i32.
+Definition core_i16_max   := i16_max %i32.
+Definition core_i32_max   := i32_max %i32.
+Definition core_i64_max   := i64_max %i64.
+Definition core_i128_max  := i64_max %i128.
+Axiom core_isize_max : isize. (** TODO *)
+
 (*** Range *)
 Record range (T : Type) := mk_range {
   start: T;
-- 
cgit v1.2.3


From 49117ba254679f98938223711810191c3f7d788f Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Fri, 27 Oct 2023 13:34:03 +0200
Subject: Regenerate the Coq test files

---
 tests/coq/hashmap_on_disk/HashmapMain_Funs.v   | 604 +++++++++++++------------
 tests/coq/hashmap_on_disk/HashmapMain_Opaque.v |   8 +-
 tests/coq/hashmap_on_disk/HashmapMain_Types.v  |  32 +-
 tests/coq/hashmap_on_disk/Primitives.v         | 405 ++++++++++++++---
 4 files changed, 675 insertions(+), 374 deletions(-)

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index a85adbf2..eac78186 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -13,652 +13,668 @@ Import HashmapMain_Opaque.
 Module HashmapMain_Funs.
 
 (** [hashmap_main::hashmap::hash_key]: forward function *)
-Definition hashmap_hash_key_fwd (k : usize) : result usize :=
+Definition hashmap_hash_key (k : usize) : result usize :=
   Return k.
 
 (** [hashmap_main::hashmap::HashMap::{0}::allocate_slots]: loop 0: forward function *)
-Fixpoint hashmap_hash_map_allocate_slots_loop_fwd
-  (T : Type) (n : nat) (slots : vec (Hashmap_list_t T)) (n0 : usize) :
-  result (vec (Hashmap_list_t T))
+Fixpoint hashmap_HashMap_allocate_slots_loop
+  (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n0 : usize)
+  :
+  result (alloc_vec_Vec (hashmap_List_t T))
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n1 =>
     if n0 s> 0%usize
     then (
-      slots0 <- vec_push_back (Hashmap_list_t T) slots HashmapListNil;
+      slots0 <- alloc_vec_Vec_push (hashmap_List_t T) slots Hashmap_List_Nil;
       n2 <- usize_sub n0 1%usize;
-      hashmap_hash_map_allocate_slots_loop_fwd T n1 slots0 n2)
+      hashmap_HashMap_allocate_slots_loop T n1 slots0 n2)
     else Return slots
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::allocate_slots]: forward function *)
-Definition hashmap_hash_map_allocate_slots_fwd
-  (T : Type) (n : nat) (slots : vec (Hashmap_list_t T)) (n0 : usize) :
-  result (vec (Hashmap_list_t T))
+Definition hashmap_HashMap_allocate_slots
+  (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n0 : usize)
+  :
+  result (alloc_vec_Vec (hashmap_List_t T))
   :=
-  hashmap_hash_map_allocate_slots_loop_fwd T n slots n0
+  hashmap_HashMap_allocate_slots_loop T n slots n0
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::new_with_capacity]: forward function *)
-Definition hashmap_hash_map_new_with_capacity_fwd
+Definition hashmap_HashMap_new_with_capacity
   (T : Type) (n : nat) (capacity : usize) (max_load_dividend : usize)
   (max_load_divisor : usize) :
-  result (Hashmap_hash_map_t T)
+  result (hashmap_HashMap_t T)
   :=
-  let v := vec_new (Hashmap_list_t T) in
-  slots <- hashmap_hash_map_allocate_slots_fwd T n v capacity;
+  let v := alloc_vec_Vec_new (hashmap_List_t T) in
+  slots <- hashmap_HashMap_allocate_slots T n v capacity;
   i <- usize_mul capacity max_load_dividend;
   i0 <- usize_div i max_load_divisor;
   Return
     {|
-      Hashmap_hash_map_num_entries := 0%usize;
-      Hashmap_hash_map_max_load_factor := (max_load_dividend, max_load_divisor);
-      Hashmap_hash_map_max_load := i0;
-      Hashmap_hash_map_slots := slots
+      hashmap_HashMap_num_entries := 0%usize;
+      hashmap_HashMap_max_load_factor := (max_load_dividend, max_load_divisor);
+      hashmap_HashMap_max_load := i0;
+      hashmap_HashMap_slots := slots
     |}
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::new]: forward function *)
-Definition hashmap_hash_map_new_fwd
-  (T : Type) (n : nat) : result (Hashmap_hash_map_t T) :=
-  hashmap_hash_map_new_with_capacity_fwd T n 32%usize 4%usize 5%usize
+Definition hashmap_HashMap_new
+  (T : Type) (n : nat) : result (hashmap_HashMap_t T) :=
+  hashmap_HashMap_new_with_capacity T n 32%usize 4%usize 5%usize
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::clear]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Fixpoint hashmap_hash_map_clear_loop_fwd_back
-  (T : Type) (n : nat) (slots : vec (Hashmap_list_t T)) (i : usize) :
-  result (vec (Hashmap_list_t T))
+Fixpoint hashmap_HashMap_clear_loop
+  (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
+  result (alloc_vec_Vec (hashmap_List_t T))
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
-    let i0 := vec_len (Hashmap_list_t T) slots in
+    let i0 := alloc_vec_Vec_len (hashmap_List_t T) slots in
     if i s< i0
     then (
       i1 <- usize_add i 1%usize;
-      slots0 <- vec_index_mut_back (Hashmap_list_t T) slots i HashmapListNil;
-      hashmap_hash_map_clear_loop_fwd_back T n0 slots0 i1)
+      slots0 <-
+        alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+          (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+          T)) slots i Hashmap_List_Nil;
+      hashmap_HashMap_clear_loop T n0 slots0 i1)
     else Return slots
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::clear]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Definition hashmap_hash_map_clear_fwd_back
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_clear
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) :
+  result (hashmap_HashMap_t T)
   :=
-  v <-
-    hashmap_hash_map_clear_loop_fwd_back T n self.(Hashmap_hash_map_slots)
-      0%usize;
+  v <- hashmap_HashMap_clear_loop T n self.(hashmap_HashMap_slots) 0%usize;
   Return
     {|
-      Hashmap_hash_map_num_entries := 0%usize;
-      Hashmap_hash_map_max_load_factor :=
-        self.(Hashmap_hash_map_max_load_factor);
-      Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-      Hashmap_hash_map_slots := v
+      hashmap_HashMap_num_entries := 0%usize;
+      hashmap_HashMap_max_load_factor := self.(hashmap_HashMap_max_load_factor);
+      hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+      hashmap_HashMap_slots := v
     |}
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::len]: forward function *)
-Definition hashmap_hash_map_len_fwd
-  (T : Type) (self : Hashmap_hash_map_t T) : result usize :=
-  Return self.(Hashmap_hash_map_num_entries)
+Definition hashmap_HashMap_len
+  (T : Type) (self : hashmap_HashMap_t T) : result usize :=
+  Return self.(hashmap_HashMap_num_entries)
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: loop 0: forward function *)
-Fixpoint hashmap_hash_map_insert_in_list_loop_fwd
-  (T : Type) (n : nat) (key : usize) (value : T) (ls : Hashmap_list_t T) :
+Fixpoint hashmap_HashMap_insert_in_list_loop
+  (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result bool
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey cvalue tl =>
+    | Hashmap_List_Cons ckey cvalue tl =>
       if ckey s= key
       then Return false
-      else hashmap_hash_map_insert_in_list_loop_fwd T n0 key value tl
-    | HashmapListNil => Return true
+      else hashmap_HashMap_insert_in_list_loop T n0 key value tl
+    | Hashmap_List_Nil => Return true
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: forward function *)
-Definition hashmap_hash_map_insert_in_list_fwd
-  (T : Type) (n : nat) (key : usize) (value : T) (ls : Hashmap_list_t T) :
+Definition hashmap_HashMap_insert_in_list
+  (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result bool
   :=
-  hashmap_hash_map_insert_in_list_loop_fwd T n key value ls
+  hashmap_HashMap_insert_in_list_loop T n key value ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: loop 0: backward function 0 *)
-Fixpoint hashmap_hash_map_insert_in_list_loop_back
-  (T : Type) (n : nat) (key : usize) (value : T) (ls : Hashmap_list_t T) :
-  result (Hashmap_list_t T)
+Fixpoint hashmap_HashMap_insert_in_list_loop_back
+  (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
+  result (hashmap_List_t T)
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey cvalue tl =>
+    | Hashmap_List_Cons ckey cvalue tl =>
       if ckey s= key
-      then Return (HashmapListCons ckey value tl)
+      then Return (Hashmap_List_Cons ckey value tl)
       else (
-        tl0 <- hashmap_hash_map_insert_in_list_loop_back T n0 key value tl;
-        Return (HashmapListCons ckey cvalue tl0))
-    | HashmapListNil =>
-      let l := HashmapListNil in Return (HashmapListCons key value l)
+        tl0 <- hashmap_HashMap_insert_in_list_loop_back T n0 key value tl;
+        Return (Hashmap_List_Cons ckey cvalue tl0))
+    | Hashmap_List_Nil =>
+      let l := Hashmap_List_Nil in Return (Hashmap_List_Cons key value l)
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: backward function 0 *)
-Definition hashmap_hash_map_insert_in_list_back
-  (T : Type) (n : nat) (key : usize) (value : T) (ls : Hashmap_list_t T) :
-  result (Hashmap_list_t T)
+Definition hashmap_HashMap_insert_in_list_back
+  (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
+  result (hashmap_List_t T)
   :=
-  hashmap_hash_map_insert_in_list_loop_back T n key value ls
+  hashmap_HashMap_insert_in_list_loop_back T n key value ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::insert_no_resize]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Definition hashmap_hash_map_insert_no_resize_fwd_back
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) (value : T)
-  :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_insert_no_resize
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (value : T) :
+  result (hashmap_HashMap_t T)
   :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
   l <-
-    vec_index_mut_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  inserted <- hashmap_hash_map_insert_in_list_fwd T n key value l;
+    alloc_vec_Vec_index_mut (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  inserted <- hashmap_HashMap_insert_in_list T n key value l;
   if inserted
   then (
-    i0 <- usize_add self.(Hashmap_hash_map_num_entries) 1%usize;
-    l0 <- hashmap_hash_map_insert_in_list_back T n key value l;
+    i0 <- usize_add self.(hashmap_HashMap_num_entries) 1%usize;
+    l0 <- hashmap_HashMap_insert_in_list_back T n key value l;
     v <-
-      vec_index_mut_back (Hashmap_list_t T) self.(Hashmap_hash_map_slots)
-        hash_mod l0;
+      alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+        T)) self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
-        Hashmap_hash_map_num_entries := i0;
-        Hashmap_hash_map_max_load_factor :=
-          self.(Hashmap_hash_map_max_load_factor);
-        Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-        Hashmap_hash_map_slots := v
+        hashmap_HashMap_num_entries := i0;
+        hashmap_HashMap_max_load_factor :=
+          self.(hashmap_HashMap_max_load_factor);
+        hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+        hashmap_HashMap_slots := v
       |})
   else (
-    l0 <- hashmap_hash_map_insert_in_list_back T n key value l;
+    l0 <- hashmap_HashMap_insert_in_list_back T n key value l;
     v <-
-      vec_index_mut_back (Hashmap_list_t T) self.(Hashmap_hash_map_slots)
-        hash_mod l0;
+      alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+        T)) self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
-        Hashmap_hash_map_num_entries := self.(Hashmap_hash_map_num_entries);
-        Hashmap_hash_map_max_load_factor :=
-          self.(Hashmap_hash_map_max_load_factor);
-        Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-        Hashmap_hash_map_slots := v
+        hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
+        hashmap_HashMap_max_load_factor :=
+          self.(hashmap_HashMap_max_load_factor);
+        hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+        hashmap_HashMap_slots := v
       |})
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::move_elements_from_list]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Fixpoint hashmap_hash_map_move_elements_from_list_loop_fwd_back
-  (T : Type) (n : nat) (ntable : Hashmap_hash_map_t T) (ls : Hashmap_list_t T)
-  :
-  result (Hashmap_hash_map_t T)
+Fixpoint hashmap_HashMap_move_elements_from_list_loop
+  (T : Type) (n : nat) (ntable : hashmap_HashMap_t T) (ls : hashmap_List_t T) :
+  result (hashmap_HashMap_t T)
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons k v tl =>
-      ntable0 <- hashmap_hash_map_insert_no_resize_fwd_back T n0 ntable k v;
-      hashmap_hash_map_move_elements_from_list_loop_fwd_back T n0 ntable0 tl
-    | HashmapListNil => Return ntable
+    | Hashmap_List_Cons k v tl =>
+      ntable0 <- hashmap_HashMap_insert_no_resize T n0 ntable k v;
+      hashmap_HashMap_move_elements_from_list_loop T n0 ntable0 tl
+    | Hashmap_List_Nil => Return ntable
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::move_elements_from_list]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Definition hashmap_hash_map_move_elements_from_list_fwd_back
-  (T : Type) (n : nat) (ntable : Hashmap_hash_map_t T) (ls : Hashmap_list_t T)
-  :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_move_elements_from_list
+  (T : Type) (n : nat) (ntable : hashmap_HashMap_t T) (ls : hashmap_List_t T) :
+  result (hashmap_HashMap_t T)
   :=
-  hashmap_hash_map_move_elements_from_list_loop_fwd_back T n ntable ls
+  hashmap_HashMap_move_elements_from_list_loop T n ntable ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::move_elements]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Fixpoint hashmap_hash_map_move_elements_loop_fwd_back
-  (T : Type) (n : nat) (ntable : Hashmap_hash_map_t T)
-  (slots : vec (Hashmap_list_t T)) (i : usize) :
-  result ((Hashmap_hash_map_t T) * (vec (Hashmap_list_t T)))
+Fixpoint hashmap_HashMap_move_elements_loop
+  (T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
+  (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
+  result ((hashmap_HashMap_t T) * (alloc_vec_Vec (hashmap_List_t T)))
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
-    let i0 := vec_len (Hashmap_list_t T) slots in
+    let i0 := alloc_vec_Vec_len (hashmap_List_t T) slots in
     if i s< i0
     then (
-      l <- vec_index_mut_fwd (Hashmap_list_t T) slots i;
-      let ls := mem_replace_fwd (Hashmap_list_t T) l HashmapListNil in
-      ntable0 <-
-        hashmap_hash_map_move_elements_from_list_fwd_back T n0 ntable ls;
+      l <-
+        alloc_vec_Vec_index_mut (hashmap_List_t T) usize
+          (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+          T)) slots i;
+      let ls := core_mem_replace (hashmap_List_t T) l Hashmap_List_Nil in
+      ntable0 <- hashmap_HashMap_move_elements_from_list T n0 ntable ls;
       i1 <- usize_add i 1%usize;
-      let l0 := mem_replace_back (Hashmap_list_t T) l HashmapListNil in
-      slots0 <- vec_index_mut_back (Hashmap_list_t T) slots i l0;
-      hashmap_hash_map_move_elements_loop_fwd_back T n0 ntable0 slots0 i1)
+      let l0 := core_mem_replace_back (hashmap_List_t T) l Hashmap_List_Nil in
+      slots0 <-
+        alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+          (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+          T)) slots i l0;
+      hashmap_HashMap_move_elements_loop T n0 ntable0 slots0 i1)
     else Return (ntable, slots)
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::move_elements]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Definition hashmap_hash_map_move_elements_fwd_back
-  (T : Type) (n : nat) (ntable : Hashmap_hash_map_t T)
-  (slots : vec (Hashmap_list_t T)) (i : usize) :
-  result ((Hashmap_hash_map_t T) * (vec (Hashmap_list_t T)))
+Definition hashmap_HashMap_move_elements
+  (T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
+  (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
+  result ((hashmap_HashMap_t T) * (alloc_vec_Vec (hashmap_List_t T)))
   :=
-  hashmap_hash_map_move_elements_loop_fwd_back T n ntable slots i
+  hashmap_HashMap_move_elements_loop T n ntable slots i
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::try_resize]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Definition hashmap_hash_map_try_resize_fwd_back
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_try_resize
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) :
+  result (hashmap_HashMap_t T)
   :=
   max_usize <- scalar_cast U32 Usize core_u32_max;
-  let capacity := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+  let capacity :=
+    alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   n1 <- usize_div max_usize 2%usize;
-  let (i, i0) := self.(Hashmap_hash_map_max_load_factor) in
+  let (i, i0) := self.(hashmap_HashMap_max_load_factor) in
   i1 <- usize_div n1 i;
   if capacity s<= i1
   then (
     i2 <- usize_mul capacity 2%usize;
-    ntable <- hashmap_hash_map_new_with_capacity_fwd T n i2 i i0;
+    ntable <- hashmap_HashMap_new_with_capacity T n i2 i i0;
     p <-
-      hashmap_hash_map_move_elements_fwd_back T n ntable
-        self.(Hashmap_hash_map_slots) 0%usize;
+      hashmap_HashMap_move_elements T n ntable self.(hashmap_HashMap_slots)
+        0%usize;
     let (ntable0, _) := p in
     Return
       {|
-        Hashmap_hash_map_num_entries := self.(Hashmap_hash_map_num_entries);
-        Hashmap_hash_map_max_load_factor := (i, i0);
-        Hashmap_hash_map_max_load := ntable0.(Hashmap_hash_map_max_load);
-        Hashmap_hash_map_slots := ntable0.(Hashmap_hash_map_slots)
+        hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
+        hashmap_HashMap_max_load_factor := (i, i0);
+        hashmap_HashMap_max_load := ntable0.(hashmap_HashMap_max_load);
+        hashmap_HashMap_slots := ntable0.(hashmap_HashMap_slots)
       |})
   else
     Return
       {|
-        Hashmap_hash_map_num_entries := self.(Hashmap_hash_map_num_entries);
-        Hashmap_hash_map_max_load_factor := (i, i0);
-        Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-        Hashmap_hash_map_slots := self.(Hashmap_hash_map_slots)
+        hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
+        hashmap_HashMap_max_load_factor := (i, i0);
+        hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+        hashmap_HashMap_slots := self.(hashmap_HashMap_slots)
       |}
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::insert]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
-Definition hashmap_hash_map_insert_fwd_back
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) (value : T)
-  :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_insert
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (value : T) :
+  result (hashmap_HashMap_t T)
   :=
-  self0 <- hashmap_hash_map_insert_no_resize_fwd_back T n self key value;
-  i <- hashmap_hash_map_len_fwd T self0;
-  if i s> self0.(Hashmap_hash_map_max_load)
-  then hashmap_hash_map_try_resize_fwd_back T n self0
+  self0 <- hashmap_HashMap_insert_no_resize T n self key value;
+  i <- hashmap_HashMap_len T self0;
+  if i s> self0.(hashmap_HashMap_max_load)
+  then hashmap_HashMap_try_resize T n self0
   else Return self0
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::contains_key_in_list]: loop 0: forward function *)
-Fixpoint hashmap_hash_map_contains_key_in_list_loop_fwd
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) : result bool :=
+Fixpoint hashmap_HashMap_contains_key_in_list_loop
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result bool :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey t tl =>
+    | Hashmap_List_Cons ckey t tl =>
       if ckey s= key
       then Return true
-      else hashmap_hash_map_contains_key_in_list_loop_fwd T n0 key tl
-    | HashmapListNil => Return false
+      else hashmap_HashMap_contains_key_in_list_loop T n0 key tl
+    | Hashmap_List_Nil => Return false
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::contains_key_in_list]: forward function *)
-Definition hashmap_hash_map_contains_key_in_list_fwd
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) : result bool :=
-  hashmap_hash_map_contains_key_in_list_loop_fwd T n key ls
+Definition hashmap_HashMap_contains_key_in_list
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result bool :=
+  hashmap_HashMap_contains_key_in_list_loop T n key ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::contains_key]: forward function *)
-Definition hashmap_hash_map_contains_key_fwd
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) :
+Definition hashmap_HashMap_contains_key
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result bool
   :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
-  l <- vec_index_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  hashmap_hash_map_contains_key_in_list_fwd T n key l
+  l <-
+    alloc_vec_Vec_index (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  hashmap_HashMap_contains_key_in_list T n key l
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_in_list]: loop 0: forward function *)
-Fixpoint hashmap_hash_map_get_in_list_loop_fwd
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) : result T :=
+Fixpoint hashmap_HashMap_get_in_list_loop
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result T :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey cvalue tl =>
+    | Hashmap_List_Cons ckey cvalue tl =>
       if ckey s= key
       then Return cvalue
-      else hashmap_hash_map_get_in_list_loop_fwd T n0 key tl
-    | HashmapListNil => Fail_ Failure
+      else hashmap_HashMap_get_in_list_loop T n0 key tl
+    | Hashmap_List_Nil => Fail_ Failure
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_in_list]: forward function *)
-Definition hashmap_hash_map_get_in_list_fwd
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) : result T :=
-  hashmap_hash_map_get_in_list_loop_fwd T n key ls
+Definition hashmap_HashMap_get_in_list
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result T :=
+  hashmap_HashMap_get_in_list_loop T n key ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get]: forward function *)
-Definition hashmap_hash_map_get_fwd
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) :
-  result T
-  :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+Definition hashmap_HashMap_get
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) : result T :=
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
-  l <- vec_index_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  hashmap_hash_map_get_in_list_fwd T n key l
+  l <-
+    alloc_vec_Vec_index (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  hashmap_HashMap_get_in_list T n key l
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: loop 0: forward function *)
-Fixpoint hashmap_hash_map_get_mut_in_list_loop_fwd
-  (T : Type) (n : nat) (ls : Hashmap_list_t T) (key : usize) : result T :=
+Fixpoint hashmap_HashMap_get_mut_in_list_loop
+  (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) : result T :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey cvalue tl =>
+    | Hashmap_List_Cons ckey cvalue tl =>
       if ckey s= key
       then Return cvalue
-      else hashmap_hash_map_get_mut_in_list_loop_fwd T n0 tl key
-    | HashmapListNil => Fail_ Failure
+      else hashmap_HashMap_get_mut_in_list_loop T n0 tl key
+    | Hashmap_List_Nil => Fail_ Failure
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: forward function *)
-Definition hashmap_hash_map_get_mut_in_list_fwd
-  (T : Type) (n : nat) (ls : Hashmap_list_t T) (key : usize) : result T :=
-  hashmap_hash_map_get_mut_in_list_loop_fwd T n ls key
+Definition hashmap_HashMap_get_mut_in_list
+  (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) : result T :=
+  hashmap_HashMap_get_mut_in_list_loop T n ls key
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: loop 0: backward function 0 *)
-Fixpoint hashmap_hash_map_get_mut_in_list_loop_back
-  (T : Type) (n : nat) (ls : Hashmap_list_t T) (key : usize) (ret : T) :
-  result (Hashmap_list_t T)
+Fixpoint hashmap_HashMap_get_mut_in_list_loop_back
+  (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) (ret : T) :
+  result (hashmap_List_t T)
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey cvalue tl =>
+    | Hashmap_List_Cons ckey cvalue tl =>
       if ckey s= key
-      then Return (HashmapListCons ckey ret tl)
+      then Return (Hashmap_List_Cons ckey ret tl)
       else (
-        tl0 <- hashmap_hash_map_get_mut_in_list_loop_back T n0 tl key ret;
-        Return (HashmapListCons ckey cvalue tl0))
-    | HashmapListNil => Fail_ Failure
+        tl0 <- hashmap_HashMap_get_mut_in_list_loop_back T n0 tl key ret;
+        Return (Hashmap_List_Cons ckey cvalue tl0))
+    | Hashmap_List_Nil => Fail_ Failure
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: backward function 0 *)
-Definition hashmap_hash_map_get_mut_in_list_back
-  (T : Type) (n : nat) (ls : Hashmap_list_t T) (key : usize) (ret : T) :
-  result (Hashmap_list_t T)
+Definition hashmap_HashMap_get_mut_in_list_back
+  (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) (ret : T) :
+  result (hashmap_List_t T)
   :=
-  hashmap_hash_map_get_mut_in_list_loop_back T n ls key ret
+  hashmap_HashMap_get_mut_in_list_loop_back T n ls key ret
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_mut]: forward function *)
-Definition hashmap_hash_map_get_mut_fwd
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) :
-  result T
-  :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+Definition hashmap_HashMap_get_mut
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) : result T :=
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
   l <-
-    vec_index_mut_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  hashmap_hash_map_get_mut_in_list_fwd T n l key
+    alloc_vec_Vec_index_mut (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  hashmap_HashMap_get_mut_in_list T n l key
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::get_mut]: backward function 0 *)
-Definition hashmap_hash_map_get_mut_back
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) (ret : T) :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_get_mut_back
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (ret : T) :
+  result (hashmap_HashMap_t T)
   :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
   l <-
-    vec_index_mut_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  l0 <- hashmap_hash_map_get_mut_in_list_back T n l key ret;
+    alloc_vec_Vec_index_mut (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  l0 <- hashmap_HashMap_get_mut_in_list_back T n l key ret;
   v <-
-    vec_index_mut_back (Hashmap_list_t T) self.(Hashmap_hash_map_slots)
-      hash_mod l0;
+    alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod l0;
   Return
     {|
-      Hashmap_hash_map_num_entries := self.(Hashmap_hash_map_num_entries);
-      Hashmap_hash_map_max_load_factor :=
-        self.(Hashmap_hash_map_max_load_factor);
-      Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-      Hashmap_hash_map_slots := v
+      hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
+      hashmap_HashMap_max_load_factor := self.(hashmap_HashMap_max_load_factor);
+      hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+      hashmap_HashMap_slots := v
     |}
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: loop 0: forward function *)
-Fixpoint hashmap_hash_map_remove_from_list_loop_fwd
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) :
+Fixpoint hashmap_HashMap_remove_from_list_loop
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (option T)
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey t tl =>
+    | Hashmap_List_Cons ckey t tl =>
       if ckey s= key
       then
         let mv_ls :=
-          mem_replace_fwd (Hashmap_list_t T) (HashmapListCons ckey t tl)
-            HashmapListNil in
+          core_mem_replace (hashmap_List_t T) (Hashmap_List_Cons ckey t tl)
+            Hashmap_List_Nil in
         match mv_ls with
-        | HashmapListCons i cvalue tl0 => Return (Some cvalue)
-        | HashmapListNil => Fail_ Failure
+        | Hashmap_List_Cons i cvalue tl0 => Return (Some cvalue)
+        | Hashmap_List_Nil => Fail_ Failure
         end
-      else hashmap_hash_map_remove_from_list_loop_fwd T n0 key tl
-    | HashmapListNil => Return None
+      else hashmap_HashMap_remove_from_list_loop T n0 key tl
+    | Hashmap_List_Nil => Return None
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: forward function *)
-Definition hashmap_hash_map_remove_from_list_fwd
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) :
+Definition hashmap_HashMap_remove_from_list
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (option T)
   :=
-  hashmap_hash_map_remove_from_list_loop_fwd T n key ls
+  hashmap_HashMap_remove_from_list_loop T n key ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: loop 0: backward function 1 *)
-Fixpoint hashmap_hash_map_remove_from_list_loop_back
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) :
-  result (Hashmap_list_t T)
+Fixpoint hashmap_HashMap_remove_from_list_loop_back
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
+  result (hashmap_List_t T)
   :=
   match n with
   | O => Fail_ OutOfFuel
   | S n0 =>
     match ls with
-    | HashmapListCons ckey t tl =>
+    | Hashmap_List_Cons ckey t tl =>
       if ckey s= key
       then
         let mv_ls :=
-          mem_replace_fwd (Hashmap_list_t T) (HashmapListCons ckey t tl)
-            HashmapListNil in
+          core_mem_replace (hashmap_List_t T) (Hashmap_List_Cons ckey t tl)
+            Hashmap_List_Nil in
         match mv_ls with
-        | HashmapListCons i cvalue tl0 => Return tl0
-        | HashmapListNil => Fail_ Failure
+        | Hashmap_List_Cons i cvalue tl0 => Return tl0
+        | Hashmap_List_Nil => Fail_ Failure
         end
       else (
-        tl0 <- hashmap_hash_map_remove_from_list_loop_back T n0 key tl;
-        Return (HashmapListCons ckey t tl0))
-    | HashmapListNil => Return HashmapListNil
+        tl0 <- hashmap_HashMap_remove_from_list_loop_back T n0 key tl;
+        Return (Hashmap_List_Cons ckey t tl0))
+    | Hashmap_List_Nil => Return Hashmap_List_Nil
     end
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: backward function 1 *)
-Definition hashmap_hash_map_remove_from_list_back
-  (T : Type) (n : nat) (key : usize) (ls : Hashmap_list_t T) :
-  result (Hashmap_list_t T)
+Definition hashmap_HashMap_remove_from_list_back
+  (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
+  result (hashmap_List_t T)
   :=
-  hashmap_hash_map_remove_from_list_loop_back T n key ls
+  hashmap_HashMap_remove_from_list_loop_back T n key ls
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::remove]: forward function *)
-Definition hashmap_hash_map_remove_fwd
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) :
+Definition hashmap_HashMap_remove
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result (option T)
   :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
   l <-
-    vec_index_mut_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  x <- hashmap_hash_map_remove_from_list_fwd T n key l;
+    alloc_vec_Vec_index_mut (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  x <- hashmap_HashMap_remove_from_list T n key l;
   match x with
   | None => Return None
   | Some x0 =>
-    _ <- usize_sub self.(Hashmap_hash_map_num_entries) 1%usize;
-    Return (Some x0)
+    _ <- usize_sub self.(hashmap_HashMap_num_entries) 1%usize; Return (Some x0)
   end
 .
 
 (** [hashmap_main::hashmap::HashMap::{0}::remove]: backward function 0 *)
-Definition hashmap_hash_map_remove_back
-  (T : Type) (n : nat) (self : Hashmap_hash_map_t T) (key : usize) :
-  result (Hashmap_hash_map_t T)
+Definition hashmap_HashMap_remove_back
+  (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
+  result (hashmap_HashMap_t T)
   :=
-  hash <- hashmap_hash_key_fwd key;
-  let i := vec_len (Hashmap_list_t T) self.(Hashmap_hash_map_slots) in
+  hash <- hashmap_hash_key key;
+  let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
   hash_mod <- usize_rem hash i;
   l <-
-    vec_index_mut_fwd (Hashmap_list_t T) self.(Hashmap_hash_map_slots) hash_mod;
-  x <- hashmap_hash_map_remove_from_list_fwd T n key l;
+    alloc_vec_Vec_index_mut (hashmap_List_t T) usize
+      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      self.(hashmap_HashMap_slots) hash_mod;
+  x <- hashmap_HashMap_remove_from_list T n key l;
   match x with
   | None =>
-    l0 <- hashmap_hash_map_remove_from_list_back T n key l;
+    l0 <- hashmap_HashMap_remove_from_list_back T n key l;
     v <-
-      vec_index_mut_back (Hashmap_list_t T) self.(Hashmap_hash_map_slots)
-        hash_mod l0;
+      alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+        T)) self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
-        Hashmap_hash_map_num_entries := self.(Hashmap_hash_map_num_entries);
-        Hashmap_hash_map_max_load_factor :=
-          self.(Hashmap_hash_map_max_load_factor);
-        Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-        Hashmap_hash_map_slots := v
+        hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
+        hashmap_HashMap_max_load_factor :=
+          self.(hashmap_HashMap_max_load_factor);
+        hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+        hashmap_HashMap_slots := v
       |}
   | Some x0 =>
-    i0 <- usize_sub self.(Hashmap_hash_map_num_entries) 1%usize;
-    l0 <- hashmap_hash_map_remove_from_list_back T n key l;
+    i0 <- usize_sub self.(hashmap_HashMap_num_entries) 1%usize;
+    l0 <- hashmap_HashMap_remove_from_list_back T n key l;
     v <-
-      vec_index_mut_back (Hashmap_list_t T) self.(Hashmap_hash_map_slots)
-        hash_mod l0;
+      alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
+        T)) self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
-        Hashmap_hash_map_num_entries := i0;
-        Hashmap_hash_map_max_load_factor :=
-          self.(Hashmap_hash_map_max_load_factor);
-        Hashmap_hash_map_max_load := self.(Hashmap_hash_map_max_load);
-        Hashmap_hash_map_slots := v
+        hashmap_HashMap_num_entries := i0;
+        hashmap_HashMap_max_load_factor :=
+          self.(hashmap_HashMap_max_load_factor);
+        hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
+        hashmap_HashMap_slots := v
       |}
   end
 .
 
 (** [hashmap_main::hashmap::test1]: forward function *)
-Definition hashmap_test1_fwd (n : nat) : result unit :=
-  hm <- hashmap_hash_map_new_fwd u64 n;
-  hm0 <- hashmap_hash_map_insert_fwd_back u64 n hm 0%usize 42%u64;
-  hm1 <- hashmap_hash_map_insert_fwd_back u64 n hm0 128%usize 18%u64;
-  hm2 <- hashmap_hash_map_insert_fwd_back u64 n hm1 1024%usize 138%u64;
-  hm3 <- hashmap_hash_map_insert_fwd_back u64 n hm2 1056%usize 256%u64;
-  i <- hashmap_hash_map_get_fwd u64 n hm3 128%usize;
+Definition hashmap_test1 (n : nat) : result unit :=
+  hm <- hashmap_HashMap_new u64 n;
+  hm0 <- hashmap_HashMap_insert u64 n hm 0%usize 42%u64;
+  hm1 <- hashmap_HashMap_insert u64 n hm0 128%usize 18%u64;
+  hm2 <- hashmap_HashMap_insert u64 n hm1 1024%usize 138%u64;
+  hm3 <- hashmap_HashMap_insert u64 n hm2 1056%usize 256%u64;
+  i <- hashmap_HashMap_get u64 n hm3 128%usize;
   if negb (i s= 18%u64)
   then Fail_ Failure
   else (
-    hm4 <- hashmap_hash_map_get_mut_back u64 n hm3 1024%usize 56%u64;
-    i0 <- hashmap_hash_map_get_fwd u64 n hm4 1024%usize;
+    hm4 <- hashmap_HashMap_get_mut_back u64 n hm3 1024%usize 56%u64;
+    i0 <- hashmap_HashMap_get u64 n hm4 1024%usize;
     if negb (i0 s= 56%u64)
     then Fail_ Failure
     else (
-      x <- hashmap_hash_map_remove_fwd u64 n hm4 1024%usize;
+      x <- hashmap_HashMap_remove u64 n hm4 1024%usize;
       match x with
       | None => Fail_ Failure
       | Some x0 =>
         if negb (x0 s= 56%u64)
         then Fail_ Failure
         else (
-          hm5 <- hashmap_hash_map_remove_back u64 n hm4 1024%usize;
-          i1 <- hashmap_hash_map_get_fwd u64 n hm5 0%usize;
+          hm5 <- hashmap_HashMap_remove_back u64 n hm4 1024%usize;
+          i1 <- hashmap_HashMap_get u64 n hm5 0%usize;
           if negb (i1 s= 42%u64)
           then Fail_ Failure
           else (
-            i2 <- hashmap_hash_map_get_fwd u64 n hm5 128%usize;
+            i2 <- hashmap_HashMap_get u64 n hm5 128%usize;
             if negb (i2 s= 18%u64)
             then Fail_ Failure
             else (
-              i3 <- hashmap_hash_map_get_fwd u64 n hm5 1056%usize;
+              i3 <- hashmap_HashMap_get u64 n hm5 1056%usize;
               if negb (i3 s= 256%u64) then Fail_ Failure else Return tt)))
       end))
 .
 
 (** [hashmap_main::insert_on_disk]: forward function *)
-Definition insert_on_disk_fwd
+Definition insert_on_disk
   (n : nat) (key : usize) (value : u64) (st : state) : result (state * unit) :=
-  p <- hashmap_utils_deserialize_fwd st;
+  p <- hashmap_utils_deserialize st;
   let (st0, hm) := p in
-  hm0 <- hashmap_hash_map_insert_fwd_back u64 n hm key value;
-  p0 <- hashmap_utils_serialize_fwd hm0 st0;
+  hm0 <- hashmap_HashMap_insert u64 n hm key value;
+  p0 <- hashmap_utils_serialize hm0 st0;
   let (st1, _) := p0 in
   Return (st1, tt)
 .
 
 (** [hashmap_main::main]: forward function *)
-Definition main_fwd : result unit :=
+Definition main : result unit :=
   Return tt.
 
-(** Unit test for [hashmap_main::main] *)
-Check (main_fwd )%return.
-
 End HashmapMain_Funs .
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v b/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
index 2d17cc29..5e376239 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
@@ -11,13 +11,13 @@ Import HashmapMain_Types.
 Module HashmapMain_Opaque.
 
 (** [hashmap_main::hashmap_utils::deserialize]: forward function *)
-Axiom hashmap_utils_deserialize_fwd
-  : state -> result (state * (Hashmap_hash_map_t u64))
+Axiom hashmap_utils_deserialize
+  : state -> result (state * (hashmap_HashMap_t u64))
 .
 
 (** [hashmap_main::hashmap_utils::serialize]: forward function *)
-Axiom hashmap_utils_serialize_fwd
-  : Hashmap_hash_map_t u64 -> state -> result (state * unit)
+Axiom hashmap_utils_serialize
+  : hashmap_HashMap_t u64 -> state -> result (state * unit)
 .
 
 End HashmapMain_Opaque .
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Types.v b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
index 36aaaf25..466119f8 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Types.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
@@ -9,29 +9,29 @@ Local Open Scope Primitives_scope.
 Module HashmapMain_Types.
 
 (** [hashmap_main::hashmap::List] *)
-Inductive Hashmap_list_t (T : Type) :=
-| HashmapListCons : usize -> T -> Hashmap_list_t T -> Hashmap_list_t T
-| HashmapListNil : Hashmap_list_t T
+Inductive hashmap_List_t (T : Type) :=
+| Hashmap_List_Cons : usize -> T -> hashmap_List_t T -> hashmap_List_t T
+| Hashmap_List_Nil : hashmap_List_t T
 .
 
-Arguments HashmapListCons {T} _ _ _.
-Arguments HashmapListNil {T}.
+Arguments Hashmap_List_Cons {T} _ _ _.
+Arguments Hashmap_List_Nil {T}.
 
 (** [hashmap_main::hashmap::HashMap] *)
-Record Hashmap_hash_map_t (T : Type) :=
-mkHashmap_hash_map_t {
-  Hashmap_hash_map_num_entries : usize;
-  Hashmap_hash_map_max_load_factor : (usize * usize);
-  Hashmap_hash_map_max_load : usize;
-  Hashmap_hash_map_slots : vec (Hashmap_list_t T);
+Record hashmap_HashMap_t (T : Type) :=
+mkhashmap_HashMap_t {
+  hashmap_HashMap_num_entries : usize;
+  hashmap_HashMap_max_load_factor : (usize * usize);
+  hashmap_HashMap_max_load : usize;
+  hashmap_HashMap_slots : alloc_vec_Vec (hashmap_List_t T);
 }
 .
 
-Arguments mkHashmap_hash_map_t {T} _ _ _ _.
-Arguments Hashmap_hash_map_num_entries {T}.
-Arguments Hashmap_hash_map_max_load_factor {T}.
-Arguments Hashmap_hash_map_max_load {T}.
-Arguments Hashmap_hash_map_slots {T}.
+Arguments mkhashmap_HashMap_t {T} _ _ _ _.
+Arguments hashmap_HashMap_num_entries {T}.
+Arguments hashmap_HashMap_max_load_factor {T}.
+Arguments hashmap_HashMap_max_load {T}.
+Arguments hashmap_HashMap_slots {T}.
 
 (** The state type used in the state-error monad *)
 Axiom state : Type.
diff --git a/tests/coq/hashmap_on_disk/Primitives.v b/tests/coq/hashmap_on_disk/Primitives.v
index 8d6c9c8d..85e38f01 100644
--- a/tests/coq/hashmap_on_disk/Primitives.v
+++ b/tests/coq/hashmap_on_disk/Primitives.v
@@ -63,13 +63,15 @@ Check (if true then Return (1 + 2) else Fail_ Failure)%global = 3.
 
 (*** Misc *)
 
-
 Definition string := Coq.Strings.String.string.
 Definition char := Coq.Strings.Ascii.ascii.
 Definition char_of_byte := Coq.Strings.Ascii.ascii_of_byte.
 
-Definition mem_replace_fwd (a : Type) (x : a) (y : a) : a := x .
-Definition mem_replace_back (a : Type) (x : a) (y : a) : a := y .
+Definition core_mem_replace (a : Type) (x : a) (y : a) : a := x .
+Definition core_mem_replace_back (a : Type) (x : a) (y : a) : a := y .
+
+Record mut_raw_ptr (T : Type) := { mut_raw_ptr_v : T }.
+Record const_raw_ptr (T : Type) := { const_raw_ptr_v : T }.
 
 (*** Scalars *)
 
@@ -408,12 +410,75 @@ Definition core_i64_max   := i64_max %i64.
 Definition core_i128_max  := i64_max %i128.
 Axiom core_isize_max : isize. (** TODO *)
 
-(*** Range *)
-Record range (T : Type) := mk_range {
-  start: T;
-  end_: T;
+(*** core::ops *)
+
+(* Trait declaration: [core::ops::index::Index] *)
+Record core_ops_index_Index (Self Idx : Type) := mk_core_ops_index_Index {
+  core_ops_index_Index_Output : Type;
+  core_ops_index_Index_index : Self -> Idx -> result core_ops_index_Index_Output;
+}.
+Arguments mk_core_ops_index_Index {_ _}.
+Arguments core_ops_index_Index_Output {_ _}.
+Arguments core_ops_index_Index_index {_ _}.
+
+(* Trait declaration: [core::ops::index::IndexMut] *)
+Record core_ops_index_IndexMut (Self Idx : Type) := mk_core_ops_index_IndexMut {
+  core_ops_index_IndexMut_indexInst : core_ops_index_Index Self Idx;
+  core_ops_index_IndexMut_index_mut : Self -> Idx -> result core_ops_index_IndexMut_indexInst.(core_ops_index_Index_Output);
+  core_ops_index_IndexMut_index_mut_back : Self -> Idx -> core_ops_index_IndexMut_indexInst.(core_ops_index_Index_Output) -> result Self;
+}.
+Arguments mk_core_ops_index_IndexMut {_ _}.
+Arguments core_ops_index_IndexMut_indexInst {_ _}.
+Arguments core_ops_index_IndexMut_index_mut {_ _}.
+Arguments core_ops_index_IndexMut_index_mut_back {_ _}.
+
+(* Trait declaration [core::ops::deref::Deref] *)
+Record core_ops_deref_Deref (Self : Type) := mk_core_ops_deref_Deref {
+  core_ops_deref_Deref_target : Type;
+  core_ops_deref_Deref_deref : Self -> result core_ops_deref_Deref_target;
+}.
+Arguments mk_core_ops_deref_Deref {_}.
+Arguments core_ops_deref_Deref_target {_}.
+Arguments core_ops_deref_Deref_deref {_}.
+
+(* Trait declaration [core::ops::deref::DerefMut] *)
+Record core_ops_deref_DerefMut (Self : Type) := mk_core_ops_deref_DerefMut {
+  core_ops_deref_DerefMut_derefInst : core_ops_deref_Deref Self;
+  core_ops_deref_DerefMut_deref_mut : Self -> result core_ops_deref_DerefMut_derefInst.(core_ops_deref_Deref_target);
+  core_ops_deref_DerefMut_deref_mut_back : Self -> core_ops_deref_DerefMut_derefInst.(core_ops_deref_Deref_target) -> result Self;
 }.
-Arguments mk_range {_}.
+Arguments mk_core_ops_deref_DerefMut {_}.
+Arguments core_ops_deref_DerefMut_derefInst {_}.
+Arguments core_ops_deref_DerefMut_deref_mut {_}.
+Arguments core_ops_deref_DerefMut_deref_mut_back {_}.
+
+Record core_ops_range_Range (T : Type) := mk_core_ops_range_Range {
+  core_ops_range_Range_start : T;
+  core_ops_range_Range_end_ : T;
+}.
+Arguments mk_core_ops_range_Range {_}.
+Arguments core_ops_range_Range_start {_}.
+Arguments core_ops_range_Range_end_ {_}.
+
+(*** [alloc] *)
+
+Definition alloc_boxed_Box_deref (T : Type) (x : T) : result T := Return x.
+Definition alloc_boxed_Box_deref_mut (T : Type) (x : T) : result T := Return x.
+Definition alloc_boxed_Box_deref_mut_back (T : Type) (_ : T) (x : T) : result T := Return x.
+
+(* Trait instance *)
+Definition alloc_boxed_Box_coreOpsDerefInst (Self : Type) : core_ops_deref_Deref Self := {|
+  core_ops_deref_Deref_target := Self;
+  core_ops_deref_Deref_deref := alloc_boxed_Box_deref Self;
+|}.
+
+(* Trait instance *)
+Definition alloc_boxed_Box_coreOpsDerefMutInst (Self : Type) : core_ops_deref_DerefMut Self := {|
+  core_ops_deref_DerefMut_derefInst := alloc_boxed_Box_coreOpsDerefInst Self;
+  core_ops_deref_DerefMut_deref_mut := alloc_boxed_Box_deref_mut Self;
+  core_ops_deref_DerefMut_deref_mut_back := alloc_boxed_Box_deref_mut_back Self;
+|}.
+
 
 (*** Arrays *)
 Definition array T (n : usize) := { l: list T | Z.of_nat (length l) = to_Z n}.
@@ -433,51 +498,50 @@ Qed.
 (* TODO: finish the definitions *)
 Axiom mk_array : forall (T : Type) (n : usize) (l : list T), array T n.
 
-Axiom array_index_shared : forall (T : Type) (n : usize) (x : array T n) (i : usize), result T.
-Axiom array_index_mut_fwd : forall (T : Type) (n : usize) (x : array T n) (i : usize), result T.
-Axiom array_index_mut_back : forall (T : Type) (n : usize) (x : array T n) (i : usize) (nx : T), result (array T n).
+(* For initialization *)
+Axiom array_repeat : forall (T : Type) (n : usize) (x : T), array T n.
+
+Axiom array_index_usize : forall (T : Type) (n : usize) (x : array T n) (i : usize), result T.
+Axiom array_update_usize : forall (T : Type) (n : usize) (x : array T n) (i : usize) (nx : T), result (array T n).
 
 (*** Slice *)
 Definition slice T := { l: list T | Z.of_nat (length l) <= usize_max}.
 
 Axiom slice_len : forall (T : Type) (s : slice T), usize.
-Axiom slice_index_shared : forall (T : Type) (x : slice T) (i : usize), result T.
-Axiom slice_index_mut_fwd : forall (T : Type) (x : slice T) (i : usize), result T.
-Axiom slice_index_mut_back : forall (T : Type) (x : slice T) (i : usize) (nx : T), result (slice T).
+Axiom slice_index_usize : forall (T : Type) (x : slice T) (i : usize), result T.
+Axiom slice_update_usize : forall (T : Type) (x : slice T) (i : usize) (nx : T), result (slice T).
 
 (*** Subslices *)
 
-Axiom array_to_slice_shared : forall (T : Type) (n : usize) (x : array T n), result (slice T).
-Axiom array_to_slice_mut_fwd : forall (T : Type) (n : usize) (x : array T n), result (slice T).
-Axiom array_to_slice_mut_back : forall (T : Type) (n : usize) (x : array T n) (s : slice T), result (array T n).
+Axiom array_to_slice : forall (T : Type) (n : usize) (x : array T n), result (slice T).
+Axiom array_from_slice : forall (T : Type) (n : usize) (x : array T n) (s : slice T), result (array T n).
+
+Axiom array_subslice: forall (T : Type) (n : usize) (x : array T n) (r : core_ops_range_Range usize), result (slice T).
+Axiom array_update_subslice: forall (T : Type) (n : usize) (x : array T n) (r : core_ops_range_Range usize) (ns : slice T), result (array T n).
 
-Axiom array_subslice_shared: forall (T : Type) (n : usize) (x : array T n) (r : range usize), result (slice T).
-Axiom array_subslice_mut_fwd: forall (T : Type) (n : usize) (x : array T n) (r : range usize), result (slice T).
-Axiom array_subslice_mut_back: forall (T : Type) (n : usize) (x : array T n) (r : range usize) (ns : slice T), result (array T n).
-Axiom slice_subslice_shared: forall (T : Type) (x : slice T) (r : range usize), result (slice T).
-Axiom slice_subslice_mut_fwd: forall (T : Type) (x : slice T) (r : range usize), result (slice T).
-Axiom slice_subslice_mut_back: forall (T : Type) (x : slice T) (r : range usize) (ns : slice T), result (slice T).
+Axiom slice_subslice: forall (T : Type) (x : slice T) (r : core_ops_range_Range usize), result (slice T).
+Axiom slice_update_subslice: forall (T : Type) (x : slice T) (r : core_ops_range_Range usize) (ns : slice T), result (slice T).
 
 (*** Vectors *)
 
-Definition vec T := { l: list T | Z.of_nat (length l) <= usize_max }.
+Definition alloc_vec_Vec T := { l: list T | Z.of_nat (length l) <= usize_max }.
 
-Definition vec_to_list {T: Type} (v: vec T) : list T := proj1_sig v.
+Definition alloc_vec_Vec_to_list {T: Type} (v: alloc_vec_Vec T) : list T := proj1_sig v.
 
-Definition vec_length {T: Type} (v: vec T) : Z := Z.of_nat (length (vec_to_list v)).
+Definition alloc_vec_Vec_length {T: Type} (v: alloc_vec_Vec T) : Z := Z.of_nat (length (alloc_vec_Vec_to_list v)).
 
-Definition vec_new (T: Type) : vec T := (exist _ [] le_0_usize_max).
+Definition alloc_vec_Vec_new (T: Type) : alloc_vec_Vec T := (exist _ [] le_0_usize_max).
 
-Lemma vec_len_in_usize {T} (v: vec T) : usize_min <= vec_length v <= usize_max.
+Lemma alloc_vec_Vec_len_in_usize {T} (v: alloc_vec_Vec T) : usize_min <= alloc_vec_Vec_length v <= usize_max.
 Proof.
-  unfold vec_length, usize_min.
+  unfold alloc_vec_Vec_length, usize_min.
   split.
   - lia.
   - apply (proj2_sig v).
 Qed.
 
-Definition vec_len (T: Type) (v: vec T) : usize :=
-  exist _ (vec_length v) (vec_len_in_usize v).
+Definition alloc_vec_Vec_len (T: Type) (v: alloc_vec_Vec T) : usize :=
+  exist _ (alloc_vec_Vec_length v) (alloc_vec_Vec_len_in_usize v).
 
 Fixpoint list_update {A} (l: list A) (n: nat) (a: A)
   : list A :=
@@ -488,50 +552,271 @@ Fixpoint list_update {A} (l: list A) (n: nat) (a: A)
     | S m => x :: (list_update t m a)
 end end.
 
-Definition vec_bind {A B} (v: vec A) (f: list A -> result (list B)) : result (vec B) :=
-  l <- f (vec_to_list v) ;
+Definition alloc_vec_Vec_bind {A B} (v: alloc_vec_Vec A) (f: list A -> result (list B)) : result (alloc_vec_Vec B) :=
+  l <- f (alloc_vec_Vec_to_list v) ;
   match sumbool_of_bool (scalar_le_max Usize (Z.of_nat (length l))) with
   | left H => Return (exist _ l (scalar_le_max_valid _ _ H))
   | right _ => Fail_ Failure
   end.
 
 (* The **forward** function shouldn't be used *)
-Definition vec_push_fwd (T: Type) (v: vec T) (x: T) : unit := tt.
+Definition alloc_vec_Vec_push_fwd (T: Type) (v: alloc_vec_Vec T) (x: T) : unit := tt.
 
-Definition vec_push_back (T: Type) (v: vec T) (x: T) : result (vec T) :=
-  vec_bind v (fun l => Return (l ++ [x])).
+Definition alloc_vec_Vec_push (T: Type) (v: alloc_vec_Vec T) (x: T) : result (alloc_vec_Vec T) :=
+  alloc_vec_Vec_bind v (fun l => Return (l ++ [x])).
 
 (* The **forward** function shouldn't be used *)
-Definition vec_insert_fwd (T: Type) (v: vec T) (i: usize) (x: T) : result unit :=
-  if to_Z i <? vec_length v then Return tt else Fail_ Failure.
+Definition alloc_vec_Vec_insert_fwd (T: Type) (v: alloc_vec_Vec T) (i: usize) (x: T) : result unit :=
+  if to_Z i <? alloc_vec_Vec_length v then Return tt else Fail_ Failure.
 
-Definition vec_insert_back (T: Type) (v: vec T) (i: usize) (x: T) : result (vec T) :=
-  vec_bind v (fun l =>
+Definition alloc_vec_Vec_insert (T: Type) (v: alloc_vec_Vec T) (i: usize) (x: T) : result (alloc_vec_Vec T) :=
+  alloc_vec_Vec_bind v (fun l =>
     if to_Z i <? Z.of_nat (length l)
     then Return (list_update l (usize_to_nat i) x)
     else Fail_ Failure).
 
-(* The **backward** function shouldn't be used *)
-Definition vec_index_fwd (T: Type) (v: vec T) (i: usize) : result T :=
-  match nth_error (vec_to_list v) (usize_to_nat i) with
-  | Some n => Return n
-  | None   => Fail_ Failure
-  end.
-
-Definition vec_index_back (T: Type) (v: vec T) (i: usize) (x: T) : result unit :=
-  if to_Z i <? vec_length v then Return tt else Fail_ Failure.
-
-(* The **backward** function shouldn't be used *)
-Definition vec_index_mut_fwd (T: Type) (v: vec T) (i: usize) : result T :=
-  match nth_error (vec_to_list v) (usize_to_nat i) with
-  | Some n => Return n
-  | None   => Fail_ Failure
+(* Helper *)
+Axiom alloc_vec_Vec_index_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : usize) (x : T), result T.
+
+(* Helper *)
+Axiom alloc_vec_Vec_update_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : usize) (x : T), result (alloc_vec_Vec T).
+
+(* Trait declaration: [core::slice::index::private_slice_index::Sealed] *)
+Definition core_slice_index_private_slice_index_Sealed (self : Type) := unit.
+
+(* Trait declaration: [core::slice::index::SliceIndex] *)
+Record core_slice_index_SliceIndex (Self T : Type) := mk_core_slice_index_SliceIndex {
+  core_slice_index_SliceIndex_sealedInst : core_slice_index_private_slice_index_Sealed Self;
+  core_slice_index_SliceIndex_Output : Type;
+  core_slice_index_SliceIndex_get : Self -> T -> result (option core_slice_index_SliceIndex_Output);
+  core_slice_index_SliceIndex_get_mut : Self -> T -> result (option core_slice_index_SliceIndex_Output);
+  core_slice_index_SliceIndex_get_mut_back : Self -> T -> option core_slice_index_SliceIndex_Output -> result T;
+  core_slice_index_SliceIndex_get_unchecked : Self -> const_raw_ptr T -> result (const_raw_ptr core_slice_index_SliceIndex_Output);
+  core_slice_index_SliceIndex_get_unchecked_mut : Self -> mut_raw_ptr T -> result (mut_raw_ptr core_slice_index_SliceIndex_Output);
+  core_slice_index_SliceIndex_index : Self -> T -> result core_slice_index_SliceIndex_Output;
+  core_slice_index_SliceIndex_index_mut : Self -> T -> result core_slice_index_SliceIndex_Output;
+  core_slice_index_SliceIndex_index_mut_back : Self -> T -> core_slice_index_SliceIndex_Output -> result T;
+}.
+Arguments mk_core_slice_index_SliceIndex {_ _}.
+Arguments core_slice_index_SliceIndex_sealedInst {_ _}.
+Arguments core_slice_index_SliceIndex_Output {_ _}.
+Arguments core_slice_index_SliceIndex_get {_ _}.
+Arguments core_slice_index_SliceIndex_get_mut {_ _}.
+Arguments core_slice_index_SliceIndex_get_mut_back {_ _}.
+Arguments core_slice_index_SliceIndex_get_unchecked {_ _}.
+Arguments core_slice_index_SliceIndex_get_unchecked_mut {_ _}.
+Arguments core_slice_index_SliceIndex_index {_ _}.
+Arguments core_slice_index_SliceIndex_index_mut {_ _}.
+Arguments core_slice_index_SliceIndex_index_mut_back {_ _}.
+
+(* [core::slice::index::[T]::index]: forward function *)
+Definition core_slice_index_Slice_index
+  (T Idx : Type) (inst : core_slice_index_SliceIndex Idx (slice T))
+  (s : slice T) (i : Idx) : result inst.(core_slice_index_SliceIndex_Output) :=
+  x <- inst.(core_slice_index_SliceIndex_get) i s;
+  match x with
+  | None => Fail_ Failure
+  | Some x => Return x
   end.
 
-Definition vec_index_mut_back (T: Type) (v: vec T) (i: usize) (x: T) : result (vec T) :=
-  vec_bind v (fun l =>
-    if to_Z i <? Z.of_nat (length l)
-    then Return (list_update l (usize_to_nat i) x)
-    else Fail_ Failure).
+(* [core::slice::index::Range:::get]: forward function *)
+Axiom core_slice_index_Range_get : forall (T : Type) (i : core_ops_range_Range usize) (s : slice T), result (option (slice T)).
+
+(* [core::slice::index::Range::get_mut]: forward function *)
+Axiom core_slice_index_Range_get_mut :
+  forall (T : Type), core_ops_range_Range usize -> slice T -> result (option (slice T)).
+
+(* [core::slice::index::Range::get_mut]: backward function 0 *)
+Axiom core_slice_index_Range_get_mut_back :
+  forall (T : Type), core_ops_range_Range usize -> slice T -> option (slice T) -> result (slice T).
+
+(* [core::slice::index::Range::get_unchecked]: forward function *)
+Definition core_slice_index_Range_get_unchecked
+  (T : Type) :
+  core_ops_range_Range usize -> const_raw_ptr (slice T) -> result (const_raw_ptr (slice T)) :=
+  (* Don't know what the model should be - for now we always fail to make
+     sure code which uses it fails *)
+  fun _ _ => Fail_ Failure.
+
+(* [core::slice::index::Range::get_unchecked_mut]: forward function *)
+Definition core_slice_index_Range_get_unchecked_mut
+  (T : Type) :
+  core_ops_range_Range usize -> mut_raw_ptr (slice T) -> result (mut_raw_ptr (slice T)) :=
+  (* Don't know what the model should be - for now we always fail to make
+    sure code which uses it fails *)
+  fun _ _ => Fail_ Failure.
+
+(* [core::slice::index::Range::index]: forward function *)
+Axiom core_slice_index_Range_index :
+  forall (T : Type), core_ops_range_Range usize -> slice T -> result (slice T).
+
+(* [core::slice::index::Range::index_mut]: forward function *)
+Axiom core_slice_index_Range_index_mut :
+  forall (T : Type), core_ops_range_Range usize -> slice T -> result (slice T).
+
+(* [core::slice::index::Range::index_mut]: backward function 0 *)
+Axiom core_slice_index_Range_index_mut_back :
+  forall (T : Type), core_ops_range_Range usize -> slice T -> slice T -> result (slice T).
+
+(* [core::slice::index::[T]::index_mut]: forward function *)
+Axiom core_slice_index_Slice_index_mut :
+  forall (T Idx : Type) (inst : core_slice_index_SliceIndex Idx (slice T)),
+  slice T -> Idx -> result inst.(core_slice_index_SliceIndex_Output).
+
+(* [core::slice::index::[T]::index_mut]: backward function 0 *)
+Axiom core_slice_index_Slice_index_mut_back :
+  forall (T Idx : Type) (inst : core_slice_index_SliceIndex Idx (slice T)),
+  slice T -> Idx -> inst.(core_slice_index_SliceIndex_Output) -> result (slice T).
+
+(* [core::array::[T; N]::index]: forward function *)
+Axiom core_array_Array_index :
+  forall (T Idx : Type) (N : usize) (inst : core_ops_index_Index (slice T) Idx)
+  (a : array T N) (i : Idx), result inst.(core_ops_index_Index_Output).
+
+(* [core::array::[T; N]::index_mut]: forward function *)
+Axiom core_array_Array_index_mut :
+  forall (T Idx : Type) (N : usize) (inst : core_ops_index_IndexMut (slice T) Idx)
+  (a : array T N) (i : Idx), result inst.(core_ops_index_IndexMut_indexInst).(core_ops_index_Index_Output).
+
+(* [core::array::[T; N]::index_mut]: backward function 0 *)
+Axiom core_array_Array_index_mut_back :
+  forall (T Idx : Type) (N : usize) (inst : core_ops_index_IndexMut (slice T) Idx)
+  (a : array T N) (i : Idx) (x : inst.(core_ops_index_IndexMut_indexInst).(core_ops_index_Index_Output)), result (array T N).
+
+(* Trait implementation: [core::slice::index::[T]] *)
+Definition core_slice_index_Slice_coreopsindexIndexInst (T Idx : Type)
+  (inst : core_slice_index_SliceIndex Idx (slice T)) :
+  core_ops_index_Index (slice T) Idx := {|
+  core_ops_index_Index_Output := inst.(core_slice_index_SliceIndex_Output);
+  core_ops_index_Index_index := core_slice_index_Slice_index T Idx inst;
+|}.
+
+(* Trait implementation: [core::slice::index::private_slice_index::Range] *)
+Definition core_slice_index_private_slice_index_Range_coresliceindexprivate_slice_indexSealedInst
+  : core_slice_index_private_slice_index_Sealed (core_ops_range_Range usize) := tt.
+
+(* Trait implementation: [core::slice::index::Range] *)
+Definition core_slice_index_Range_coresliceindexSliceIndexInst (T : Type) :
+  core_slice_index_SliceIndex (core_ops_range_Range usize) (slice T) := {|
+  core_slice_index_SliceIndex_sealedInst := core_slice_index_private_slice_index_Range_coresliceindexprivate_slice_indexSealedInst;
+  core_slice_index_SliceIndex_Output := slice T;
+  core_slice_index_SliceIndex_get := core_slice_index_Range_get T;
+  core_slice_index_SliceIndex_get_mut := core_slice_index_Range_get_mut T;
+  core_slice_index_SliceIndex_get_mut_back := core_slice_index_Range_get_mut_back T;
+  core_slice_index_SliceIndex_get_unchecked := core_slice_index_Range_get_unchecked T;
+  core_slice_index_SliceIndex_get_unchecked_mut := core_slice_index_Range_get_unchecked_mut T;
+  core_slice_index_SliceIndex_index := core_slice_index_Range_index T;
+  core_slice_index_SliceIndex_index_mut := core_slice_index_Range_index_mut T;
+  core_slice_index_SliceIndex_index_mut_back := core_slice_index_Range_index_mut_back T;
+|}.
+
+(* Trait implementation: [core::slice::index::[T]] *)
+Definition core_slice_index_Slice_coreopsindexIndexMutInst (T Idx : Type)
+  (inst : core_slice_index_SliceIndex Idx (slice T)) :
+  core_ops_index_IndexMut (slice T) Idx := {|
+  core_ops_index_IndexMut_indexInst := core_slice_index_Slice_coreopsindexIndexInst T Idx inst;
+  core_ops_index_IndexMut_index_mut := core_slice_index_Slice_index_mut T Idx inst;
+  core_ops_index_IndexMut_index_mut_back := core_slice_index_Slice_index_mut_back T Idx inst;
+|}.
+
+(* Trait implementation: [core::array::[T; N]] *)
+Definition core_array_Array_coreopsindexIndexInst (T Idx : Type) (N : usize)
+  (inst : core_ops_index_Index (slice T) Idx) :
+  core_ops_index_Index (array T N) Idx := {|
+  core_ops_index_Index_Output := inst.(core_ops_index_Index_Output);
+  core_ops_index_Index_index := core_array_Array_index T Idx N inst;
+|}.
+
+(* Trait implementation: [core::array::[T; N]] *)
+Definition core_array_Array_coreopsindexIndexMutInst (T Idx : Type) (N : usize)
+  (inst : core_ops_index_IndexMut (slice T) Idx) :
+  core_ops_index_IndexMut (array T N) Idx := {|
+  core_ops_index_IndexMut_indexInst := core_array_Array_coreopsindexIndexInst T Idx N inst.(core_ops_index_IndexMut_indexInst);
+  core_ops_index_IndexMut_index_mut := core_array_Array_index_mut T Idx N inst;
+  core_ops_index_IndexMut_index_mut_back := core_array_Array_index_mut_back T Idx N inst;
+|}.
+
+(* [core::slice::index::usize::get]: forward function *)
+Axiom core_slice_index_usize_get : forall (T : Type), usize -> slice T -> result (option T).
+
+(* [core::slice::index::usize::get_mut]: forward function *)
+Axiom core_slice_index_usize_get_mut : forall (T : Type), usize -> slice T -> result (option T).
+
+(* [core::slice::index::usize::get_mut]: backward function 0 *)
+Axiom core_slice_index_usize_get_mut_back :
+  forall (T : Type), usize -> slice T -> option T -> result (slice T).
+
+(* [core::slice::index::usize::get_unchecked]: forward function *)
+Axiom core_slice_index_usize_get_unchecked :
+  forall (T : Type), usize -> const_raw_ptr (slice T) -> result (const_raw_ptr T).
+
+(* [core::slice::index::usize::get_unchecked_mut]: forward function *)
+Axiom core_slice_index_usize_get_unchecked_mut :
+  forall (T : Type), usize -> mut_raw_ptr (slice T) -> result (mut_raw_ptr T).
+
+(* [core::slice::index::usize::index]: forward function *)
+Axiom core_slice_index_usize_index : forall (T : Type), usize -> slice T -> result T.
+
+(* [core::slice::index::usize::index_mut]: forward function *)
+Axiom core_slice_index_usize_index_mut : forall (T : Type), usize -> slice T -> result T.
+
+(* [core::slice::index::usize::index_mut]: backward function 0 *)
+Axiom core_slice_index_usize_index_mut_back :
+  forall (T : Type), usize -> slice T -> T -> result (slice T).
+
+(* Trait implementation: [core::slice::index::private_slice_index::usize] *)
+Definition core_slice_index_private_slice_index_usize_coresliceindexprivate_slice_indexSealedInst
+  : core_slice_index_private_slice_index_Sealed usize := tt.
+
+(* Trait implementation: [core::slice::index::usize] *)
+Definition core_slice_index_usize_coresliceindexSliceIndexInst (T : Type) :
+  core_slice_index_SliceIndex usize (slice T) := {|
+  core_slice_index_SliceIndex_sealedInst := core_slice_index_private_slice_index_usize_coresliceindexprivate_slice_indexSealedInst;
+  core_slice_index_SliceIndex_Output := T;
+  core_slice_index_SliceIndex_get := core_slice_index_usize_get T;
+  core_slice_index_SliceIndex_get_mut := core_slice_index_usize_get_mut T;
+  core_slice_index_SliceIndex_get_mut_back := core_slice_index_usize_get_mut_back T;
+  core_slice_index_SliceIndex_get_unchecked := core_slice_index_usize_get_unchecked T;
+  core_slice_index_SliceIndex_get_unchecked_mut := core_slice_index_usize_get_unchecked_mut T;
+  core_slice_index_SliceIndex_index := core_slice_index_usize_index T;
+  core_slice_index_SliceIndex_index_mut := core_slice_index_usize_index_mut T;
+  core_slice_index_SliceIndex_index_mut_back := core_slice_index_usize_index_mut_back T;
+|}.
+
+(* [alloc::vec::Vec::index]: forward function *)
+Axiom alloc_vec_Vec_index : forall (T Idx : Type) (inst : core_slice_index_SliceIndex Idx (slice T))
+  (Self : alloc_vec_Vec T) (i : Idx), result inst.(core_slice_index_SliceIndex_Output).
+
+(* [alloc::vec::Vec::index_mut]: forward function *)
+Axiom alloc_vec_Vec_index_mut : forall (T Idx : Type) (inst : core_slice_index_SliceIndex Idx (slice T))
+  (Self : alloc_vec_Vec T) (i : Idx), result inst.(core_slice_index_SliceIndex_Output).
+
+(* [alloc::vec::Vec::index_mut]: backward function 0 *)
+Axiom alloc_vec_Vec_index_mut_back :
+  forall (T Idx : Type) (inst : core_slice_index_SliceIndex Idx (slice T))
+  (Self : alloc_vec_Vec T) (i : Idx) (x : inst.(core_slice_index_SliceIndex_Output)), result (alloc_vec_Vec T).
+
+(* Trait implementation: [alloc::vec::Vec] *)
+Definition alloc_vec_Vec_coreopsindexIndexInst (T Idx : Type)
+  (inst : core_slice_index_SliceIndex Idx (slice T)) :
+  core_ops_index_Index (alloc_vec_Vec T) Idx := {|
+  core_ops_index_Index_Output := inst.(core_slice_index_SliceIndex_Output);
+  core_ops_index_Index_index := alloc_vec_Vec_index T Idx inst;
+|}.
+
+(* Trait implementation: [alloc::vec::Vec] *)
+Definition alloc_vec_Vec_coreopsindexIndexMutInst (T Idx : Type)
+  (inst : core_slice_index_SliceIndex Idx (slice T)) :
+  core_ops_index_IndexMut (alloc_vec_Vec T) Idx := {|
+  core_ops_index_IndexMut_indexInst := alloc_vec_Vec_coreopsindexIndexInst T Idx inst;
+  core_ops_index_IndexMut_index_mut := alloc_vec_Vec_index_mut T Idx inst;
+  core_ops_index_IndexMut_index_mut_back := alloc_vec_Vec_index_mut_back T Idx inst;
+|}.
+
+(*** Theorems *)
+
+Axiom alloc_vec_Vec_index_mut_back_eq : forall {a : Type} (v : alloc_vec_Vec a) (i : usize) (x : a),
+  alloc_vec_Vec_index_mut_back a usize (core_slice_index_usize_coresliceindexSliceIndexInst a) v i x =
+    alloc_vec_Vec_update_usize v i x.
 
 End Primitives.
-- 
cgit v1.2.3


From 49ffc966cfdbd71f8c83a3c72ab81e1bb101f420 Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Thu, 9 Nov 2023 16:24:07 +0100
Subject: Regenerate the Coq test files

---
 tests/coq/hashmap_on_disk/HashmapMain_Types.v | 14 +++++++-------
 1 file changed, 7 insertions(+), 7 deletions(-)

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Types.v b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
index 466119f8..95e5f35b 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Types.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
@@ -14,8 +14,8 @@ Inductive hashmap_List_t (T : Type) :=
 | Hashmap_List_Nil : hashmap_List_t T
 .
 
-Arguments Hashmap_List_Cons {T} _ _ _.
-Arguments Hashmap_List_Nil {T}.
+Arguments Hashmap_List_Cons { _ }.
+Arguments Hashmap_List_Nil { _ }.
 
 (** [hashmap_main::hashmap::HashMap] *)
 Record hashmap_HashMap_t (T : Type) :=
@@ -27,11 +27,11 @@ mkhashmap_HashMap_t {
 }
 .
 
-Arguments mkhashmap_HashMap_t {T} _ _ _ _.
-Arguments hashmap_HashMap_num_entries {T}.
-Arguments hashmap_HashMap_max_load_factor {T}.
-Arguments hashmap_HashMap_max_load {T}.
-Arguments hashmap_HashMap_slots {T}.
+Arguments mkhashmap_HashMap_t { _ }.
+Arguments hashmap_HashMap_num_entries { _ }.
+Arguments hashmap_HashMap_max_load_factor { _ }.
+Arguments hashmap_HashMap_max_load { _ }.
+Arguments hashmap_HashMap_slots { _ }.
 
 (** The state type used in the state-error monad *)
 Axiom state : Type.
-- 
cgit v1.2.3


From 5e92ae6b361f9221f5c5f9a39ab4c28a36597a77 Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Tue, 21 Nov 2023 11:40:59 +0100
Subject: Regenerate most of the test files

---
 tests/coq/hashmap_on_disk/HashmapMain_Funs.v | 116 +++++++++++++--------------
 tests/coq/hashmap_on_disk/Primitives.v       |  88 +++++++++++---------
 2 files changed, 106 insertions(+), 98 deletions(-)

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index eac78186..6f3848e6 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -16,7 +16,7 @@ Module HashmapMain_Funs.
 Definition hashmap_hash_key (k : usize) : result usize :=
   Return k.
 
-(** [hashmap_main::hashmap::HashMap::{0}::allocate_slots]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: loop 0: forward function *)
 Fixpoint hashmap_HashMap_allocate_slots_loop
   (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n0 : usize)
   :
@@ -34,7 +34,7 @@ Fixpoint hashmap_HashMap_allocate_slots_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::allocate_slots]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: forward function *)
 Definition hashmap_HashMap_allocate_slots
   (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n0 : usize)
   :
@@ -43,7 +43,7 @@ Definition hashmap_HashMap_allocate_slots
   hashmap_HashMap_allocate_slots_loop T n slots n0
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::new_with_capacity]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new_with_capacity]: forward function *)
 Definition hashmap_HashMap_new_with_capacity
   (T : Type) (n : nat) (capacity : usize) (max_load_dividend : usize)
   (max_load_divisor : usize) :
@@ -62,13 +62,13 @@ Definition hashmap_HashMap_new_with_capacity
     |}
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::new]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new]: forward function *)
 Definition hashmap_HashMap_new
   (T : Type) (n : nat) : result (hashmap_HashMap_t T) :=
   hashmap_HashMap_new_with_capacity T n 32%usize 4%usize 5%usize
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::clear]: loop 0: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Fixpoint hashmap_HashMap_clear_loop
   (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
@@ -83,14 +83,14 @@ Fixpoint hashmap_HashMap_clear_loop
       i1 <- usize_add i 1%usize;
       slots0 <-
         alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-          (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-          T)) slots i Hashmap_List_Nil;
+          (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T)) slots
+          i Hashmap_List_Nil;
       hashmap_HashMap_clear_loop T n0 slots0 i1)
     else Return slots
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::clear]: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Definition hashmap_HashMap_clear
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) :
@@ -106,13 +106,13 @@ Definition hashmap_HashMap_clear
     |}
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::len]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::len]: forward function *)
 Definition hashmap_HashMap_len
   (T : Type) (self : hashmap_HashMap_t T) : result usize :=
   Return self.(hashmap_HashMap_num_entries)
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: loop 0: forward function *)
 Fixpoint hashmap_HashMap_insert_in_list_loop
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result bool
@@ -130,7 +130,7 @@ Fixpoint hashmap_HashMap_insert_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: forward function *)
 Definition hashmap_HashMap_insert_in_list
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result bool
@@ -138,7 +138,7 @@ Definition hashmap_HashMap_insert_in_list
   hashmap_HashMap_insert_in_list_loop T n key value ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: loop 0: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: loop 0: backward function 0 *)
 Fixpoint hashmap_HashMap_insert_in_list_loop_back
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -159,7 +159,7 @@ Fixpoint hashmap_HashMap_insert_in_list_loop_back
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::insert_in_list]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: backward function 0 *)
 Definition hashmap_HashMap_insert_in_list_back
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -167,7 +167,7 @@ Definition hashmap_HashMap_insert_in_list_back
   hashmap_HashMap_insert_in_list_loop_back T n key value ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::insert_no_resize]: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_no_resize]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Definition hashmap_HashMap_insert_no_resize
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (value : T) :
@@ -178,7 +178,7 @@ Definition hashmap_HashMap_insert_no_resize
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index_mut (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   inserted <- hashmap_HashMap_insert_in_list T n key value l;
   if inserted
@@ -187,8 +187,8 @@ Definition hashmap_HashMap_insert_no_resize
     l0 <- hashmap_HashMap_insert_in_list_back T n key value l;
     v <-
       alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-        T)) self.(hashmap_HashMap_slots) hash_mod l0;
+        (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
+        self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
         hashmap_HashMap_num_entries := i0;
@@ -201,8 +201,8 @@ Definition hashmap_HashMap_insert_no_resize
     l0 <- hashmap_HashMap_insert_in_list_back T n key value l;
     v <-
       alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-        T)) self.(hashmap_HashMap_slots) hash_mod l0;
+        (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
+        self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
         hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
@@ -213,7 +213,7 @@ Definition hashmap_HashMap_insert_no_resize
       |})
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::move_elements_from_list]: loop 0: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements_from_list]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Fixpoint hashmap_HashMap_move_elements_from_list_loop
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T) (ls : hashmap_List_t T) :
@@ -231,7 +231,7 @@ Fixpoint hashmap_HashMap_move_elements_from_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::move_elements_from_list]: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements_from_list]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Definition hashmap_HashMap_move_elements_from_list
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T) (ls : hashmap_List_t T) :
@@ -240,7 +240,7 @@ Definition hashmap_HashMap_move_elements_from_list
   hashmap_HashMap_move_elements_from_list_loop T n ntable ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::move_elements]: loop 0: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements]: loop 0: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Fixpoint hashmap_HashMap_move_elements_loop
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
@@ -255,22 +255,22 @@ Fixpoint hashmap_HashMap_move_elements_loop
     then (
       l <-
         alloc_vec_Vec_index_mut (hashmap_List_t T) usize
-          (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-          T)) slots i;
+          (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T)) slots
+          i;
       let ls := core_mem_replace (hashmap_List_t T) l Hashmap_List_Nil in
       ntable0 <- hashmap_HashMap_move_elements_from_list T n0 ntable ls;
       i1 <- usize_add i 1%usize;
       let l0 := core_mem_replace_back (hashmap_List_t T) l Hashmap_List_Nil in
       slots0 <-
         alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-          (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-          T)) slots i l0;
+          (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T)) slots
+          i l0;
       hashmap_HashMap_move_elements_loop T n0 ntable0 slots0 i1)
     else Return (ntable, slots)
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::move_elements]: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Definition hashmap_HashMap_move_elements
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
@@ -280,7 +280,7 @@ Definition hashmap_HashMap_move_elements
   hashmap_HashMap_move_elements_loop T n ntable slots i
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::try_resize]: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::try_resize]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Definition hashmap_HashMap_try_resize
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) :
@@ -317,7 +317,7 @@ Definition hashmap_HashMap_try_resize
       |}
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::insert]: merged forward/backward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert]: merged forward/backward function
     (there is a single backward function, and the forward function returns ()) *)
 Definition hashmap_HashMap_insert
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (value : T) :
@@ -330,7 +330,7 @@ Definition hashmap_HashMap_insert
   else Return self0
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::contains_key_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key_in_list]: loop 0: forward function *)
 Fixpoint hashmap_HashMap_contains_key_in_list_loop
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result bool :=
   match n with
@@ -346,13 +346,13 @@ Fixpoint hashmap_HashMap_contains_key_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::contains_key_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key_in_list]: forward function *)
 Definition hashmap_HashMap_contains_key_in_list
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result bool :=
   hashmap_HashMap_contains_key_in_list_loop T n key ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::contains_key]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key]: forward function *)
 Definition hashmap_HashMap_contains_key
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result bool
@@ -362,12 +362,12 @@ Definition hashmap_HashMap_contains_key
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   hashmap_HashMap_contains_key_in_list T n key l
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_in_list]: loop 0: forward function *)
 Fixpoint hashmap_HashMap_get_in_list_loop
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result T :=
   match n with
@@ -383,13 +383,13 @@ Fixpoint hashmap_HashMap_get_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_in_list]: forward function *)
 Definition hashmap_HashMap_get_in_list
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result T :=
   hashmap_HashMap_get_in_list_loop T n key ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get]: forward function *)
 Definition hashmap_HashMap_get
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) : result T :=
   hash <- hashmap_hash_key key;
@@ -397,12 +397,12 @@ Definition hashmap_HashMap_get
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   hashmap_HashMap_get_in_list T n key l
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: loop 0: forward function *)
 Fixpoint hashmap_HashMap_get_mut_in_list_loop
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) : result T :=
   match n with
@@ -418,13 +418,13 @@ Fixpoint hashmap_HashMap_get_mut_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: forward function *)
 Definition hashmap_HashMap_get_mut_in_list
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) : result T :=
   hashmap_HashMap_get_mut_in_list_loop T n ls key
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: loop 0: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: loop 0: backward function 0 *)
 Fixpoint hashmap_HashMap_get_mut_in_list_loop_back
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) (ret : T) :
   result (hashmap_List_t T)
@@ -444,7 +444,7 @@ Fixpoint hashmap_HashMap_get_mut_in_list_loop_back
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_mut_in_list]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: backward function 0 *)
 Definition hashmap_HashMap_get_mut_in_list_back
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) (ret : T) :
   result (hashmap_List_t T)
@@ -452,7 +452,7 @@ Definition hashmap_HashMap_get_mut_in_list_back
   hashmap_HashMap_get_mut_in_list_loop_back T n ls key ret
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_mut]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: forward function *)
 Definition hashmap_HashMap_get_mut
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) : result T :=
   hash <- hashmap_hash_key key;
@@ -460,12 +460,12 @@ Definition hashmap_HashMap_get_mut
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index_mut (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   hashmap_HashMap_get_mut_in_list T n l key
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::get_mut]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: backward function 0 *)
 Definition hashmap_HashMap_get_mut_back
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (ret : T) :
   result (hashmap_HashMap_t T)
@@ -475,12 +475,12 @@ Definition hashmap_HashMap_get_mut_back
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index_mut (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   l0 <- hashmap_HashMap_get_mut_in_list_back T n l key ret;
   v <-
     alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod l0;
   Return
     {|
@@ -491,7 +491,7 @@ Definition hashmap_HashMap_get_mut_back
     |}
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: forward function *)
 Fixpoint hashmap_HashMap_remove_from_list_loop
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (option T)
@@ -516,7 +516,7 @@ Fixpoint hashmap_HashMap_remove_from_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: forward function *)
 Definition hashmap_HashMap_remove_from_list
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (option T)
@@ -524,7 +524,7 @@ Definition hashmap_HashMap_remove_from_list
   hashmap_HashMap_remove_from_list_loop T n key ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: loop 0: backward function 1 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: backward function 1 *)
 Fixpoint hashmap_HashMap_remove_from_list_loop_back
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -551,7 +551,7 @@ Fixpoint hashmap_HashMap_remove_from_list_loop_back
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::remove_from_list]: backward function 1 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: backward function 1 *)
 Definition hashmap_HashMap_remove_from_list_back
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -559,7 +559,7 @@ Definition hashmap_HashMap_remove_from_list_back
   hashmap_HashMap_remove_from_list_loop_back T n key ls
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::remove]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove]: forward function *)
 Definition hashmap_HashMap_remove
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result (option T)
@@ -569,7 +569,7 @@ Definition hashmap_HashMap_remove
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index_mut (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   x <- hashmap_HashMap_remove_from_list T n key l;
   match x with
@@ -579,7 +579,7 @@ Definition hashmap_HashMap_remove
   end
 .
 
-(** [hashmap_main::hashmap::HashMap::{0}::remove]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove]: backward function 0 *)
 Definition hashmap_HashMap_remove_back
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result (hashmap_HashMap_t T)
@@ -589,7 +589,7 @@ Definition hashmap_HashMap_remove_back
   hash_mod <- usize_rem hash i;
   l <-
     alloc_vec_Vec_index_mut (hashmap_List_t T) usize
-      (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t T))
+      (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
       self.(hashmap_HashMap_slots) hash_mod;
   x <- hashmap_HashMap_remove_from_list T n key l;
   match x with
@@ -597,8 +597,8 @@ Definition hashmap_HashMap_remove_back
     l0 <- hashmap_HashMap_remove_from_list_back T n key l;
     v <-
       alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-        T)) self.(hashmap_HashMap_slots) hash_mod l0;
+        (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
+        self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
         hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
@@ -612,8 +612,8 @@ Definition hashmap_HashMap_remove_back
     l0 <- hashmap_HashMap_remove_from_list_back T n key l;
     v <-
       alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
-        (core_slice_index_usize_coresliceindexSliceIndexInst (hashmap_List_t
-        T)) self.(hashmap_HashMap_slots) hash_mod l0;
+        (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
+        self.(hashmap_HashMap_slots) hash_mod l0;
     Return
       {|
         hashmap_HashMap_num_entries := i0;
diff --git a/tests/coq/hashmap_on_disk/Primitives.v b/tests/coq/hashmap_on_disk/Primitives.v
index 85e38f01..83f860b6 100644
--- a/tests/coq/hashmap_on_disk/Primitives.v
+++ b/tests/coq/hashmap_on_disk/Primitives.v
@@ -467,14 +467,14 @@ Definition alloc_boxed_Box_deref_mut (T : Type) (x : T) : result T := Return x.
 Definition alloc_boxed_Box_deref_mut_back (T : Type) (_ : T) (x : T) : result T := Return x.
 
 (* Trait instance *)
-Definition alloc_boxed_Box_coreOpsDerefInst (Self : Type) : core_ops_deref_Deref Self := {|
+Definition alloc_boxed_Box_coreopsDerefInst (Self : Type) : core_ops_deref_Deref Self := {|
   core_ops_deref_Deref_target := Self;
   core_ops_deref_Deref_deref := alloc_boxed_Box_deref Self;
 |}.
 
 (* Trait instance *)
-Definition alloc_boxed_Box_coreOpsDerefMutInst (Self : Type) : core_ops_deref_DerefMut Self := {|
-  core_ops_deref_DerefMut_derefInst := alloc_boxed_Box_coreOpsDerefInst Self;
+Definition alloc_boxed_Box_coreopsDerefMutInst (Self : Type) : core_ops_deref_DerefMut Self := {|
+  core_ops_deref_DerefMut_derefInst := alloc_boxed_Box_coreopsDerefInst Self;
   core_ops_deref_DerefMut_deref_mut := alloc_boxed_Box_deref_mut Self;
   core_ops_deref_DerefMut_deref_mut_back := alloc_boxed_Box_deref_mut_back Self;
 |}.
@@ -576,7 +576,7 @@ Definition alloc_vec_Vec_insert (T: Type) (v: alloc_vec_Vec T) (i: usize) (x: T)
     else Fail_ Failure).
 
 (* Helper *)
-Axiom alloc_vec_Vec_index_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : usize) (x : T), result T.
+Axiom alloc_vec_Vec_index_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : usize), result T.
 
 (* Helper *)
 Axiom alloc_vec_Vec_update_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : usize) (x : T), result (alloc_vec_Vec T).
@@ -620,18 +620,18 @@ Definition core_slice_index_Slice_index
   end.
 
 (* [core::slice::index::Range:::get]: forward function *)
-Axiom core_slice_index_Range_get : forall (T : Type) (i : core_ops_range_Range usize) (s : slice T), result (option (slice T)).
+Axiom core_slice_index_RangeUsize_get : forall (T : Type) (i : core_ops_range_Range usize) (s : slice T), result (option (slice T)).
 
 (* [core::slice::index::Range::get_mut]: forward function *)
-Axiom core_slice_index_Range_get_mut :
+Axiom core_slice_index_RangeUsize_get_mut :
   forall (T : Type), core_ops_range_Range usize -> slice T -> result (option (slice T)).
 
 (* [core::slice::index::Range::get_mut]: backward function 0 *)
-Axiom core_slice_index_Range_get_mut_back :
+Axiom core_slice_index_RangeUsize_get_mut_back :
   forall (T : Type), core_ops_range_Range usize -> slice T -> option (slice T) -> result (slice T).
 
 (* [core::slice::index::Range::get_unchecked]: forward function *)
-Definition core_slice_index_Range_get_unchecked
+Definition core_slice_index_RangeUsize_get_unchecked
   (T : Type) :
   core_ops_range_Range usize -> const_raw_ptr (slice T) -> result (const_raw_ptr (slice T)) :=
   (* Don't know what the model should be - for now we always fail to make
@@ -639,7 +639,7 @@ Definition core_slice_index_Range_get_unchecked
   fun _ _ => Fail_ Failure.
 
 (* [core::slice::index::Range::get_unchecked_mut]: forward function *)
-Definition core_slice_index_Range_get_unchecked_mut
+Definition core_slice_index_RangeUsize_get_unchecked_mut
   (T : Type) :
   core_ops_range_Range usize -> mut_raw_ptr (slice T) -> result (mut_raw_ptr (slice T)) :=
   (* Don't know what the model should be - for now we always fail to make
@@ -647,15 +647,15 @@ Definition core_slice_index_Range_get_unchecked_mut
   fun _ _ => Fail_ Failure.
 
 (* [core::slice::index::Range::index]: forward function *)
-Axiom core_slice_index_Range_index :
+Axiom core_slice_index_RangeUsize_index :
   forall (T : Type), core_ops_range_Range usize -> slice T -> result (slice T).
 
 (* [core::slice::index::Range::index_mut]: forward function *)
-Axiom core_slice_index_Range_index_mut :
+Axiom core_slice_index_RangeUsize_index_mut :
   forall (T : Type), core_ops_range_Range usize -> slice T -> result (slice T).
 
 (* [core::slice::index::Range::index_mut]: backward function 0 *)
-Axiom core_slice_index_Range_index_mut_back :
+Axiom core_slice_index_RangeUsize_index_mut_back :
   forall (T : Type), core_ops_range_Range usize -> slice T -> slice T -> result (slice T).
 
 (* [core::slice::index::[T]::index_mut]: forward function *)
@@ -683,44 +683,44 @@ Axiom core_array_Array_index_mut_back :
   forall (T Idx : Type) (N : usize) (inst : core_ops_index_IndexMut (slice T) Idx)
   (a : array T N) (i : Idx) (x : inst.(core_ops_index_IndexMut_indexInst).(core_ops_index_Index_Output)), result (array T N).
 
-(* Trait implementation: [core::slice::index::[T]] *)
-Definition core_slice_index_Slice_coreopsindexIndexInst (T Idx : Type)
-  (inst : core_slice_index_SliceIndex Idx (slice T)) :
-  core_ops_index_Index (slice T) Idx := {|
-  core_ops_index_Index_Output := inst.(core_slice_index_SliceIndex_Output);
-  core_ops_index_Index_index := core_slice_index_Slice_index T Idx inst;
-|}.
-
 (* Trait implementation: [core::slice::index::private_slice_index::Range] *)
-Definition core_slice_index_private_slice_index_Range_coresliceindexprivate_slice_indexSealedInst
+Definition core_slice_index_private_slice_index_SealedRangeUsizeInst
   : core_slice_index_private_slice_index_Sealed (core_ops_range_Range usize) := tt.
 
 (* Trait implementation: [core::slice::index::Range] *)
-Definition core_slice_index_Range_coresliceindexSliceIndexInst (T : Type) :
+Definition core_slice_index_SliceIndexRangeUsizeSliceTInst (T : Type) :
   core_slice_index_SliceIndex (core_ops_range_Range usize) (slice T) := {|
-  core_slice_index_SliceIndex_sealedInst := core_slice_index_private_slice_index_Range_coresliceindexprivate_slice_indexSealedInst;
+  core_slice_index_SliceIndex_sealedInst := core_slice_index_private_slice_index_SealedRangeUsizeInst;
   core_slice_index_SliceIndex_Output := slice T;
-  core_slice_index_SliceIndex_get := core_slice_index_Range_get T;
-  core_slice_index_SliceIndex_get_mut := core_slice_index_Range_get_mut T;
-  core_slice_index_SliceIndex_get_mut_back := core_slice_index_Range_get_mut_back T;
-  core_slice_index_SliceIndex_get_unchecked := core_slice_index_Range_get_unchecked T;
-  core_slice_index_SliceIndex_get_unchecked_mut := core_slice_index_Range_get_unchecked_mut T;
-  core_slice_index_SliceIndex_index := core_slice_index_Range_index T;
-  core_slice_index_SliceIndex_index_mut := core_slice_index_Range_index_mut T;
-  core_slice_index_SliceIndex_index_mut_back := core_slice_index_Range_index_mut_back T;
+  core_slice_index_SliceIndex_get := core_slice_index_RangeUsize_get T;
+  core_slice_index_SliceIndex_get_mut := core_slice_index_RangeUsize_get_mut T;
+  core_slice_index_SliceIndex_get_mut_back := core_slice_index_RangeUsize_get_mut_back T;
+  core_slice_index_SliceIndex_get_unchecked := core_slice_index_RangeUsize_get_unchecked T;
+  core_slice_index_SliceIndex_get_unchecked_mut := core_slice_index_RangeUsize_get_unchecked_mut T;
+  core_slice_index_SliceIndex_index := core_slice_index_RangeUsize_index T;
+  core_slice_index_SliceIndex_index_mut := core_slice_index_RangeUsize_index_mut T;
+  core_slice_index_SliceIndex_index_mut_back := core_slice_index_RangeUsize_index_mut_back T;
+|}.
+
+(* Trait implementation: [core::slice::index::[T]] *)
+Definition core_ops_index_IndexSliceTIInst (T Idx : Type)
+  (inst : core_slice_index_SliceIndex Idx (slice T)) :
+  core_ops_index_Index (slice T) Idx := {|
+  core_ops_index_Index_Output := inst.(core_slice_index_SliceIndex_Output);
+  core_ops_index_Index_index := core_slice_index_Slice_index T Idx inst;
 |}.
 
 (* Trait implementation: [core::slice::index::[T]] *)
-Definition core_slice_index_Slice_coreopsindexIndexMutInst (T Idx : Type)
+Definition core_ops_index_IndexMutSliceTIInst (T Idx : Type)
   (inst : core_slice_index_SliceIndex Idx (slice T)) :
   core_ops_index_IndexMut (slice T) Idx := {|
-  core_ops_index_IndexMut_indexInst := core_slice_index_Slice_coreopsindexIndexInst T Idx inst;
+  core_ops_index_IndexMut_indexInst := core_ops_index_IndexSliceTIInst T Idx inst;
   core_ops_index_IndexMut_index_mut := core_slice_index_Slice_index_mut T Idx inst;
   core_ops_index_IndexMut_index_mut_back := core_slice_index_Slice_index_mut_back T Idx inst;
 |}.
 
 (* Trait implementation: [core::array::[T; N]] *)
-Definition core_array_Array_coreopsindexIndexInst (T Idx : Type) (N : usize)
+Definition core_ops_index_IndexArrayInst (T Idx : Type) (N : usize)
   (inst : core_ops_index_Index (slice T) Idx) :
   core_ops_index_Index (array T N) Idx := {|
   core_ops_index_Index_Output := inst.(core_ops_index_Index_Output);
@@ -728,10 +728,10 @@ Definition core_array_Array_coreopsindexIndexInst (T Idx : Type) (N : usize)
 |}.
 
 (* Trait implementation: [core::array::[T; N]] *)
-Definition core_array_Array_coreopsindexIndexMutInst (T Idx : Type) (N : usize)
+Definition core_ops_index_IndexMutArrayInst (T Idx : Type) (N : usize)
   (inst : core_ops_index_IndexMut (slice T) Idx) :
   core_ops_index_IndexMut (array T N) Idx := {|
-  core_ops_index_IndexMut_indexInst := core_array_Array_coreopsindexIndexInst T Idx N inst.(core_ops_index_IndexMut_indexInst);
+  core_ops_index_IndexMut_indexInst := core_ops_index_IndexArrayInst T Idx N inst.(core_ops_index_IndexMut_indexInst);
   core_ops_index_IndexMut_index_mut := core_array_Array_index_mut T Idx N inst;
   core_ops_index_IndexMut_index_mut_back := core_array_Array_index_mut_back T Idx N inst;
 |}.
@@ -765,13 +765,13 @@ Axiom core_slice_index_usize_index_mut_back :
   forall (T : Type), usize -> slice T -> T -> result (slice T).
 
 (* Trait implementation: [core::slice::index::private_slice_index::usize] *)
-Definition core_slice_index_private_slice_index_usize_coresliceindexprivate_slice_indexSealedInst
+Definition core_slice_index_private_slice_index_SealedUsizeInst
   : core_slice_index_private_slice_index_Sealed usize := tt.
 
 (* Trait implementation: [core::slice::index::usize] *)
-Definition core_slice_index_usize_coresliceindexSliceIndexInst (T : Type) :
+Definition core_slice_index_SliceIndexUsizeSliceTInst (T : Type) :
   core_slice_index_SliceIndex usize (slice T) := {|
-  core_slice_index_SliceIndex_sealedInst := core_slice_index_private_slice_index_usize_coresliceindexprivate_slice_indexSealedInst;
+  core_slice_index_SliceIndex_sealedInst := core_slice_index_private_slice_index_SealedUsizeInst;
   core_slice_index_SliceIndex_Output := T;
   core_slice_index_SliceIndex_get := core_slice_index_usize_get T;
   core_slice_index_SliceIndex_get_mut := core_slice_index_usize_get_mut T;
@@ -815,8 +815,16 @@ Definition alloc_vec_Vec_coreopsindexIndexMutInst (T Idx : Type)
 
 (*** Theorems *)
 
+Axiom alloc_vec_Vec_index_eq : forall {a : Type} (v : alloc_vec_Vec a) (i : usize) (x : a),
+  alloc_vec_Vec_index a usize (core_slice_index_SliceIndexUsizeSliceTInst a) v i =
+    alloc_vec_Vec_index_usize v i.
+
+Axiom alloc_vec_Vec_index_mut_eq : forall {a : Type} (v : alloc_vec_Vec a) (i : usize) (x : a),
+  alloc_vec_Vec_index_mut a usize (core_slice_index_SliceIndexUsizeSliceTInst a) v i =
+    alloc_vec_Vec_index_usize v i.
+
 Axiom alloc_vec_Vec_index_mut_back_eq : forall {a : Type} (v : alloc_vec_Vec a) (i : usize) (x : a),
-  alloc_vec_Vec_index_mut_back a usize (core_slice_index_usize_coresliceindexSliceIndexInst a) v i x =
+  alloc_vec_Vec_index_mut_back a usize (core_slice_index_SliceIndexUsizeSliceTInst a) v i x =
     alloc_vec_Vec_update_usize v i x.
 
 End Primitives.
-- 
cgit v1.2.3


From 137cc7335e64fcb70c254e7fd2a6fa353fb43e61 Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Tue, 21 Nov 2023 14:57:38 +0100
Subject: Regenerate the files

---
 tests/coq/hashmap_on_disk/HashmapMain_Funs.v   | 120 ++++++++++++++++---------
 tests/coq/hashmap_on_disk/HashmapMain_Opaque.v |   6 +-
 tests/coq/hashmap_on_disk/HashmapMain_Types.v  |   6 +-
 3 files changed, 88 insertions(+), 44 deletions(-)

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index 6f3848e6..46d3ee29 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -12,11 +12,13 @@ Require Export HashmapMain_Opaque.
 Import HashmapMain_Opaque.
 Module HashmapMain_Funs.
 
-(** [hashmap_main::hashmap::hash_key]: forward function *)
+(** [hashmap_main::hashmap::hash_key]: forward function
+    Source: 'src/hashmap.rs', lines 27:0-27:32 *)
 Definition hashmap_hash_key (k : usize) : result usize :=
   Return k.
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: loop 0: forward function
+    Source: 'src/hashmap.rs', lines 50:4-56:5 *)
 Fixpoint hashmap_HashMap_allocate_slots_loop
   (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n0 : usize)
   :
@@ -34,7 +36,8 @@ Fixpoint hashmap_HashMap_allocate_slots_loop
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: forward function
+    Source: 'src/hashmap.rs', lines 50:4-50:76 *)
 Definition hashmap_HashMap_allocate_slots
   (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n0 : usize)
   :
@@ -43,7 +46,8 @@ Definition hashmap_HashMap_allocate_slots
   hashmap_HashMap_allocate_slots_loop T n slots n0
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new_with_capacity]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new_with_capacity]: forward function
+    Source: 'src/hashmap.rs', lines 59:4-63:13 *)
 Definition hashmap_HashMap_new_with_capacity
   (T : Type) (n : nat) (capacity : usize) (max_load_dividend : usize)
   (max_load_divisor : usize) :
@@ -62,14 +66,16 @@ Definition hashmap_HashMap_new_with_capacity
     |}
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new]: forward function
+    Source: 'src/hashmap.rs', lines 75:4-75:24 *)
 Definition hashmap_HashMap_new
   (T : Type) (n : nat) : result (hashmap_HashMap_t T) :=
   hashmap_HashMap_new_with_capacity T n 32%usize 4%usize 5%usize
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]: loop 0: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 80:4-88:5 *)
 Fixpoint hashmap_HashMap_clear_loop
   (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
   result (alloc_vec_Vec (hashmap_List_t T))
@@ -91,7 +97,8 @@ Fixpoint hashmap_HashMap_clear_loop
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 80:4-80:27 *)
 Definition hashmap_HashMap_clear
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) :
   result (hashmap_HashMap_t T)
@@ -106,13 +113,15 @@ Definition hashmap_HashMap_clear
     |}
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::len]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::len]: forward function
+    Source: 'src/hashmap.rs', lines 90:4-90:30 *)
 Definition hashmap_HashMap_len
   (T : Type) (self : hashmap_HashMap_t T) : result usize :=
   Return self.(hashmap_HashMap_num_entries)
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: loop 0: forward function
+    Source: 'src/hashmap.rs', lines 97:4-114:5 *)
 Fixpoint hashmap_HashMap_insert_in_list_loop
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result bool
@@ -130,7 +139,8 @@ Fixpoint hashmap_HashMap_insert_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: forward function
+    Source: 'src/hashmap.rs', lines 97:4-97:71 *)
 Definition hashmap_HashMap_insert_in_list
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result bool
@@ -138,7 +148,8 @@ Definition hashmap_HashMap_insert_in_list
   hashmap_HashMap_insert_in_list_loop T n key value ls
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: loop 0: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: loop 0: backward function 0
+    Source: 'src/hashmap.rs', lines 97:4-114:5 *)
 Fixpoint hashmap_HashMap_insert_in_list_loop_back
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -159,7 +170,8 @@ Fixpoint hashmap_HashMap_insert_in_list_loop_back
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_in_list]: backward function 0
+    Source: 'src/hashmap.rs', lines 97:4-97:71 *)
 Definition hashmap_HashMap_insert_in_list_back
   (T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -168,7 +180,8 @@ Definition hashmap_HashMap_insert_in_list_back
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_no_resize]: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 117:4-117:54 *)
 Definition hashmap_HashMap_insert_no_resize
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (value : T) :
   result (hashmap_HashMap_t T)
@@ -214,7 +227,8 @@ Definition hashmap_HashMap_insert_no_resize
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements_from_list]: loop 0: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 183:4-196:5 *)
 Fixpoint hashmap_HashMap_move_elements_from_list_loop
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T) (ls : hashmap_List_t T) :
   result (hashmap_HashMap_t T)
@@ -232,7 +246,8 @@ Fixpoint hashmap_HashMap_move_elements_from_list_loop
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements_from_list]: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 183:4-183:72 *)
 Definition hashmap_HashMap_move_elements_from_list
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T) (ls : hashmap_List_t T) :
   result (hashmap_HashMap_t T)
@@ -241,7 +256,8 @@ Definition hashmap_HashMap_move_elements_from_list
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements]: loop 0: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 171:4-180:5 *)
 Fixpoint hashmap_HashMap_move_elements_loop
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
   (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
@@ -271,7 +287,8 @@ Fixpoint hashmap_HashMap_move_elements_loop
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements]: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 171:4-171:95 *)
 Definition hashmap_HashMap_move_elements
   (T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
   (slots : alloc_vec_Vec (hashmap_List_t T)) (i : usize) :
@@ -281,7 +298,8 @@ Definition hashmap_HashMap_move_elements
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::try_resize]: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 140:4-140:28 *)
 Definition hashmap_HashMap_try_resize
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) :
   result (hashmap_HashMap_t T)
@@ -318,7 +336,8 @@ Definition hashmap_HashMap_try_resize
 .
 
 (** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert]: merged forward/backward function
-    (there is a single backward function, and the forward function returns ()) *)
+    (there is a single backward function, and the forward function returns ())
+    Source: 'src/hashmap.rs', lines 129:4-129:48 *)
 Definition hashmap_HashMap_insert
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (value : T) :
   result (hashmap_HashMap_t T)
@@ -330,7 +349,8 @@ Definition hashmap_HashMap_insert
   else Return self0
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key_in_list]: loop 0: forward function
+    Source: 'src/hashmap.rs', lines 206:4-219:5 *)
 Fixpoint hashmap_HashMap_contains_key_in_list_loop
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result bool :=
   match n with
@@ -346,13 +366,15 @@ Fixpoint hashmap_HashMap_contains_key_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key_in_list]: forward function
+    Source: 'src/hashmap.rs', lines 206:4-206:68 *)
 Definition hashmap_HashMap_contains_key_in_list
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result bool :=
   hashmap_HashMap_contains_key_in_list_loop T n key ls
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::contains_key]: forward function
+    Source: 'src/hashmap.rs', lines 199:4-199:49 *)
 Definition hashmap_HashMap_contains_key
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result bool
@@ -367,7 +389,8 @@ Definition hashmap_HashMap_contains_key
   hashmap_HashMap_contains_key_in_list T n key l
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_in_list]: loop 0: forward function
+    Source: 'src/hashmap.rs', lines 224:4-237:5 *)
 Fixpoint hashmap_HashMap_get_in_list_loop
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result T :=
   match n with
@@ -383,13 +406,15 @@ Fixpoint hashmap_HashMap_get_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_in_list]: forward function
+    Source: 'src/hashmap.rs', lines 224:4-224:70 *)
 Definition hashmap_HashMap_get_in_list
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) : result T :=
   hashmap_HashMap_get_in_list_loop T n key ls
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get]: forward function
+    Source: 'src/hashmap.rs', lines 239:4-239:55 *)
 Definition hashmap_HashMap_get
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) : result T :=
   hash <- hashmap_hash_key key;
@@ -402,7 +427,8 @@ Definition hashmap_HashMap_get
   hashmap_HashMap_get_in_list T n key l
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: loop 0: forward function
+    Source: 'src/hashmap.rs', lines 245:4-254:5 *)
 Fixpoint hashmap_HashMap_get_mut_in_list_loop
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) : result T :=
   match n with
@@ -418,13 +444,15 @@ Fixpoint hashmap_HashMap_get_mut_in_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: forward function
+    Source: 'src/hashmap.rs', lines 245:4-245:86 *)
 Definition hashmap_HashMap_get_mut_in_list
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) : result T :=
   hashmap_HashMap_get_mut_in_list_loop T n ls key
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: loop 0: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: loop 0: backward function 0
+    Source: 'src/hashmap.rs', lines 245:4-254:5 *)
 Fixpoint hashmap_HashMap_get_mut_in_list_loop_back
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) (ret : T) :
   result (hashmap_List_t T)
@@ -444,7 +472,8 @@ Fixpoint hashmap_HashMap_get_mut_in_list_loop_back
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut_in_list]: backward function 0
+    Source: 'src/hashmap.rs', lines 245:4-245:86 *)
 Definition hashmap_HashMap_get_mut_in_list_back
   (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) (ret : T) :
   result (hashmap_List_t T)
@@ -452,7 +481,8 @@ Definition hashmap_HashMap_get_mut_in_list_back
   hashmap_HashMap_get_mut_in_list_loop_back T n ls key ret
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: forward function
+    Source: 'src/hashmap.rs', lines 257:4-257:67 *)
 Definition hashmap_HashMap_get_mut
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) : result T :=
   hash <- hashmap_hash_key key;
@@ -465,7 +495,8 @@ Definition hashmap_HashMap_get_mut
   hashmap_HashMap_get_mut_in_list T n l key
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: backward function 0
+    Source: 'src/hashmap.rs', lines 257:4-257:67 *)
 Definition hashmap_HashMap_get_mut_back
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) (ret : T) :
   result (hashmap_HashMap_t T)
@@ -491,7 +522,8 @@ Definition hashmap_HashMap_get_mut_back
     |}
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: forward function
+    Source: 'src/hashmap.rs', lines 265:4-291:5 *)
 Fixpoint hashmap_HashMap_remove_from_list_loop
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (option T)
@@ -516,7 +548,8 @@ Fixpoint hashmap_HashMap_remove_from_list_loop
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: forward function
+    Source: 'src/hashmap.rs', lines 265:4-265:69 *)
 Definition hashmap_HashMap_remove_from_list
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (option T)
@@ -524,7 +557,8 @@ Definition hashmap_HashMap_remove_from_list
   hashmap_HashMap_remove_from_list_loop T n key ls
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: backward function 1 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: backward function 1
+    Source: 'src/hashmap.rs', lines 265:4-291:5 *)
 Fixpoint hashmap_HashMap_remove_from_list_loop_back
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -551,7 +585,8 @@ Fixpoint hashmap_HashMap_remove_from_list_loop_back
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: backward function 1 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: backward function 1
+    Source: 'src/hashmap.rs', lines 265:4-265:69 *)
 Definition hashmap_HashMap_remove_from_list_back
   (T : Type) (n : nat) (key : usize) (ls : hashmap_List_t T) :
   result (hashmap_List_t T)
@@ -559,7 +594,8 @@ Definition hashmap_HashMap_remove_from_list_back
   hashmap_HashMap_remove_from_list_loop_back T n key ls
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove]: forward function *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove]: forward function
+    Source: 'src/hashmap.rs', lines 294:4-294:52 *)
 Definition hashmap_HashMap_remove
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result (option T)
@@ -579,7 +615,8 @@ Definition hashmap_HashMap_remove
   end
 .
 
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove]: backward function 0 *)
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove]: backward function 0
+    Source: 'src/hashmap.rs', lines 294:4-294:52 *)
 Definition hashmap_HashMap_remove_back
   (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
   result (hashmap_HashMap_t T)
@@ -625,7 +662,8 @@ Definition hashmap_HashMap_remove_back
   end
 .
 
-(** [hashmap_main::hashmap::test1]: forward function *)
+(** [hashmap_main::hashmap::test1]: forward function
+    Source: 'src/hashmap.rs', lines 315:0-315:10 *)
 Definition hashmap_test1 (n : nat) : result unit :=
   hm <- hashmap_HashMap_new u64 n;
   hm0 <- hashmap_HashMap_insert u64 n hm 0%usize 42%u64;
@@ -662,7 +700,8 @@ Definition hashmap_test1 (n : nat) : result unit :=
       end))
 .
 
-(** [hashmap_main::insert_on_disk]: forward function *)
+(** [hashmap_main::insert_on_disk]: forward function
+    Source: 'src/hashmap_main.rs', lines 7:0-7:43 *)
 Definition insert_on_disk
   (n : nat) (key : usize) (value : u64) (st : state) : result (state * unit) :=
   p <- hashmap_utils_deserialize st;
@@ -673,7 +712,8 @@ Definition insert_on_disk
   Return (st1, tt)
 .
 
-(** [hashmap_main::main]: forward function *)
+(** [hashmap_main::main]: forward function
+    Source: 'src/hashmap_main.rs', lines 16:0-16:13 *)
 Definition main : result unit :=
   Return tt.
 
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v b/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
index 5e376239..a0e9003d 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
@@ -10,12 +10,14 @@ Require Export HashmapMain_Types.
 Import HashmapMain_Types.
 Module HashmapMain_Opaque.
 
-(** [hashmap_main::hashmap_utils::deserialize]: forward function *)
+(** [hashmap_main::hashmap_utils::deserialize]: forward function
+    Source: 'src/hashmap_utils.rs', lines 10:0-10:43 *)
 Axiom hashmap_utils_deserialize
   : state -> result (state * (hashmap_HashMap_t u64))
 .
 
-(** [hashmap_main::hashmap_utils::serialize]: forward function *)
+(** [hashmap_main::hashmap_utils::serialize]: forward function
+    Source: 'src/hashmap_utils.rs', lines 5:0-5:42 *)
 Axiom hashmap_utils_serialize
   : hashmap_HashMap_t u64 -> state -> result (state * unit)
 .
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Types.v b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
index 95e5f35b..039b7e72 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Types.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
@@ -8,7 +8,8 @@ Import ListNotations.
 Local Open Scope Primitives_scope.
 Module HashmapMain_Types.
 
-(** [hashmap_main::hashmap::List] *)
+(** [hashmap_main::hashmap::List]
+    Source: 'src/hashmap.rs', lines 19:0-19:16 *)
 Inductive hashmap_List_t (T : Type) :=
 | Hashmap_List_Cons : usize -> T -> hashmap_List_t T -> hashmap_List_t T
 | Hashmap_List_Nil : hashmap_List_t T
@@ -17,7 +18,8 @@ Inductive hashmap_List_t (T : Type) :=
 Arguments Hashmap_List_Cons { _ }.
 Arguments Hashmap_List_Nil { _ }.
 
-(** [hashmap_main::hashmap::HashMap] *)
+(** [hashmap_main::hashmap::HashMap]
+    Source: 'src/hashmap.rs', lines 35:0-35:21 *)
 Record hashmap_HashMap_t (T : Type) :=
 mkhashmap_HashMap_t {
   hashmap_HashMap_num_entries : usize;
-- 
cgit v1.2.3


From 959d6fce38c8d8ca6eaed3ad6f458b87f91a9abc Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Mon, 27 Nov 2023 09:37:31 +0100
Subject: Update the generation of files for external definitions and
 regenerate the tests

---
 tests/coq/hashmap_on_disk/HashmapMain_Funs.v       |  4 ++--
 .../coq/hashmap_on_disk/HashmapMain_FunsExternal.v | 25 +++++++++++++++++++++
 .../HashmapMain_FunsExternal_Template.v            | 26 ++++++++++++++++++++++
 tests/coq/hashmap_on_disk/HashmapMain_Opaque.v     | 25 ---------------------
 tests/coq/hashmap_on_disk/_CoqProject              |  3 ++-
 5 files changed, 55 insertions(+), 28 deletions(-)
 create mode 100644 tests/coq/hashmap_on_disk/HashmapMain_FunsExternal.v
 create mode 100644 tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
 delete mode 100644 tests/coq/hashmap_on_disk/HashmapMain_Opaque.v

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index 46d3ee29..188c98b3 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -8,8 +8,8 @@ Import ListNotations.
 Local Open Scope Primitives_scope.
 Require Export HashmapMain_Types.
 Import HashmapMain_Types.
-Require Export HashmapMain_Opaque.
-Import HashmapMain_Opaque.
+Require Export HashmapMain_FunsExternal.
+Import HashmapMain_FunsExternal.
 Module HashmapMain_Funs.
 
 (** [hashmap_main::hashmap::hash_key]: forward function
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal.v b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal.v
new file mode 100644
index 00000000..a03dc407
--- /dev/null
+++ b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal.v
@@ -0,0 +1,25 @@
+(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
+(** [hashmap_main]: external function declarations *)
+Require Import Primitives.
+Import Primitives.
+Require Import Coq.ZArith.ZArith.
+Require Import List.
+Import ListNotations.
+Local Open Scope Primitives_scope.
+Require Export HashmapMain_Types.
+Import HashmapMain_Types.
+Module HashmapMain_FunsExternal.
+
+(** [hashmap_main::hashmap_utils::deserialize]: forward function
+    Source: 'src/hashmap_utils.rs', lines 10:0-10:43 *)
+Axiom hashmap_utils_deserialize
+  : state -> result (state * (hashmap_HashMap_t u64))
+.
+
+(** [hashmap_main::hashmap_utils::serialize]: forward function
+    Source: 'src/hashmap_utils.rs', lines 5:0-5:42 *)
+Axiom hashmap_utils_serialize
+  : hashmap_HashMap_t u64 -> state -> result (state * unit)
+.
+
+End HashmapMain_FunsExternal.
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
new file mode 100644
index 00000000..b5a4a101
--- /dev/null
+++ b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
@@ -0,0 +1,26 @@
+(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
+(** [hashmap_main]: external functions.
+-- This is a template file: rename it to "FunsExternal.lean" and fill the holes. *)
+Require Import Primitives.
+Import Primitives.
+Require Import Coq.ZArith.ZArith.
+Require Import List.
+Import ListNotations.
+Local Open Scope Primitives_scope.
+Require Export HashmapMain_Types.
+Import HashmapMain_Types.
+Module HashmapMain_FunsExternal_Template.
+
+(** [hashmap_main::hashmap_utils::deserialize]: forward function
+    Source: 'src/hashmap_utils.rs', lines 10:0-10:43 *)
+Axiom hashmap_utils_deserialize
+  : state -> result (state * (hashmap_HashMap_t u64))
+.
+
+(** [hashmap_main::hashmap_utils::serialize]: forward function
+    Source: 'src/hashmap_utils.rs', lines 5:0-5:42 *)
+Axiom hashmap_utils_serialize
+  : hashmap_HashMap_t u64 -> state -> result (state * unit)
+.
+
+End HashmapMain_FunsExternal_Template .
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v b/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
deleted file mode 100644
index a0e9003d..00000000
--- a/tests/coq/hashmap_on_disk/HashmapMain_Opaque.v
+++ /dev/null
@@ -1,25 +0,0 @@
-(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
-(** [hashmap_main]: external function declarations *)
-Require Import Primitives.
-Import Primitives.
-Require Import Coq.ZArith.ZArith.
-Require Import List.
-Import ListNotations.
-Local Open Scope Primitives_scope.
-Require Export HashmapMain_Types.
-Import HashmapMain_Types.
-Module HashmapMain_Opaque.
-
-(** [hashmap_main::hashmap_utils::deserialize]: forward function
-    Source: 'src/hashmap_utils.rs', lines 10:0-10:43 *)
-Axiom hashmap_utils_deserialize
-  : state -> result (state * (hashmap_HashMap_t u64))
-.
-
-(** [hashmap_main::hashmap_utils::serialize]: forward function
-    Source: 'src/hashmap_utils.rs', lines 5:0-5:42 *)
-Axiom hashmap_utils_serialize
-  : hashmap_HashMap_t u64 -> state -> result (state * unit)
-.
-
-End HashmapMain_Opaque .
diff --git a/tests/coq/hashmap_on_disk/_CoqProject b/tests/coq/hashmap_on_disk/_CoqProject
index b78c7b5f..a85fa1fe 100644
--- a/tests/coq/hashmap_on_disk/_CoqProject
+++ b/tests/coq/hashmap_on_disk/_CoqProject
@@ -6,4 +6,5 @@
 HashmapMain_Types.v
 Primitives.v
 HashmapMain_Funs.v
-HashmapMain_Opaque.v
+HashmapMain_FunsExternal_Template.v
+HashmapMain_FunsExternal.v
-- 
cgit v1.2.3


From bef2bd34fcb0817f1b7d16b95122bcc3c6f05c72 Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Mon, 27 Nov 2023 10:29:25 +0100
Subject: Generate a dedicated file for the external types

---
 tests/coq/hashmap_on_disk/HashmapMain_Funs.v              | 10 +++++-----
 .../hashmap_on_disk/HashmapMain_FunsExternal_Template.v   |  6 +++---
 tests/coq/hashmap_on_disk/HashmapMain_Types.v             |  7 +++----
 tests/coq/hashmap_on_disk/HashmapMain_TypesExternal.v     | 15 +++++++++++++++
 .../hashmap_on_disk/HashmapMain_TypesExternal_Template.v  | 15 +++++++++++++++
 tests/coq/hashmap_on_disk/_CoqProject                     |  2 ++
 6 files changed, 43 insertions(+), 12 deletions(-)
 create mode 100644 tests/coq/hashmap_on_disk/HashmapMain_TypesExternal.v
 create mode 100644 tests/coq/hashmap_on_disk/HashmapMain_TypesExternal_Template.v

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index 188c98b3..faba0afe 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -6,10 +6,10 @@ Require Import Coq.ZArith.ZArith.
 Require Import List.
 Import ListNotations.
 Local Open Scope Primitives_scope.
-Require Export HashmapMain_Types.
-Import HashmapMain_Types.
-Require Export HashmapMain_FunsExternal.
-Import HashmapMain_FunsExternal.
+Require Import HashmapMain_Types.
+Include HashmapMain_Types.
+Require Import HashmapMain_FunsExternal.
+Include HashmapMain_FunsExternal.
 Module HashmapMain_Funs.
 
 (** [hashmap_main::hashmap::hash_key]: forward function
@@ -717,4 +717,4 @@ Definition insert_on_disk
 Definition main : result unit :=
   Return tt.
 
-End HashmapMain_Funs .
+End HashmapMain_Funs.
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
index b5a4a101..e10d02f6 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
@@ -7,8 +7,8 @@ Require Import Coq.ZArith.ZArith.
 Require Import List.
 Import ListNotations.
 Local Open Scope Primitives_scope.
-Require Export HashmapMain_Types.
-Import HashmapMain_Types.
+Require Import HashmapMain_Types.
+Include HashmapMain_Types.
 Module HashmapMain_FunsExternal_Template.
 
 (** [hashmap_main::hashmap_utils::deserialize]: forward function
@@ -23,4 +23,4 @@ Axiom hashmap_utils_serialize
   : hashmap_HashMap_t u64 -> state -> result (state * unit)
 .
 
-End HashmapMain_FunsExternal_Template .
+End HashmapMain_FunsExternal_Template.
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Types.v b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
index 039b7e72..8d3d72aa 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Types.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Types.v
@@ -6,6 +6,8 @@ Require Import Coq.ZArith.ZArith.
 Require Import List.
 Import ListNotations.
 Local Open Scope Primitives_scope.
+Require Import HashmapMain_TypesExternal.
+Include HashmapMain_TypesExternal.
 Module HashmapMain_Types.
 
 (** [hashmap_main::hashmap::List]
@@ -35,7 +37,4 @@ Arguments hashmap_HashMap_max_load_factor { _ }.
 Arguments hashmap_HashMap_max_load { _ }.
 Arguments hashmap_HashMap_slots { _ }.
 
-(** The state type used in the state-error monad *)
-Axiom state : Type.
-
-End HashmapMain_Types .
+End HashmapMain_Types.
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_TypesExternal.v b/tests/coq/hashmap_on_disk/HashmapMain_TypesExternal.v
new file mode 100644
index 00000000..87568232
--- /dev/null
+++ b/tests/coq/hashmap_on_disk/HashmapMain_TypesExternal.v
@@ -0,0 +1,15 @@
+(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
+(** [hashmap_main]: external types.
+-- This is a template file: rename it to "TypesExternal.lean" and fill the holes. *)
+Require Import Primitives.
+Import Primitives.
+Require Import Coq.ZArith.ZArith.
+Require Import List.
+Import ListNotations.
+Local Open Scope Primitives_scope.
+Module HashmapMain_TypesExternal.
+
+(** The state type used in the state-error monad *)
+Axiom state : Type.
+
+End HashmapMain_TypesExternal.
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_TypesExternal_Template.v b/tests/coq/hashmap_on_disk/HashmapMain_TypesExternal_Template.v
new file mode 100644
index 00000000..391b2775
--- /dev/null
+++ b/tests/coq/hashmap_on_disk/HashmapMain_TypesExternal_Template.v
@@ -0,0 +1,15 @@
+(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
+(** [hashmap_main]: external types.
+-- This is a template file: rename it to "TypesExternal.lean" and fill the holes. *)
+Require Import Primitives.
+Import Primitives.
+Require Import Coq.ZArith.ZArith.
+Require Import List.
+Import ListNotations.
+Local Open Scope Primitives_scope.
+Module HashmapMain_TypesExternal_Template.
+
+(** The state type used in the state-error monad *)
+Axiom state : Type.
+
+End HashmapMain_TypesExternal_Template.
diff --git a/tests/coq/hashmap_on_disk/_CoqProject b/tests/coq/hashmap_on_disk/_CoqProject
index a85fa1fe..41945494 100644
--- a/tests/coq/hashmap_on_disk/_CoqProject
+++ b/tests/coq/hashmap_on_disk/_CoqProject
@@ -6,5 +6,7 @@
 HashmapMain_Types.v
 Primitives.v
 HashmapMain_Funs.v
+HashmapMain_TypesExternal.v
 HashmapMain_FunsExternal_Template.v
 HashmapMain_FunsExternal.v
+HashmapMain_TypesExternal_Template.v
-- 
cgit v1.2.3


From 3b487893b2906e13b2388efc3512f2babc8514bf Mon Sep 17 00:00:00 2001
From: Son Ho
Date: Wed, 29 Nov 2023 15:48:27 +0100
Subject: Regenerate the other files

---
 tests/coq/hashmap_on_disk/Primitives.v | 76 ++++++++++++++++++++++++++++++++++
 1 file changed, 76 insertions(+)

(limited to 'tests/coq/hashmap_on_disk')

diff --git a/tests/coq/hashmap_on_disk/Primitives.v b/tests/coq/hashmap_on_disk/Primitives.v
index 83f860b6..99ffe070 100644
--- a/tests/coq/hashmap_on_disk/Primitives.v
+++ b/tests/coq/hashmap_on_disk/Primitives.v
@@ -255,6 +255,12 @@ Definition scalar_rem {ty} (x y: scalar ty) : result (scalar ty) := mk_scalar ty
   
 Definition scalar_neg {ty} (x: scalar ty) : result (scalar ty) := mk_scalar ty (-(to_Z x)).
 
+Axiom scalar_xor : forall ty, scalar ty -> scalar ty -> scalar ty. (* TODO *)
+Axiom scalar_or : forall ty, scalar ty -> scalar ty -> scalar ty. (* TODO *)
+Axiom scalar_and : forall ty, scalar ty -> scalar ty -> scalar ty. (* TODO *)
+Axiom scalar_shl : forall ty0 ty1, scalar ty0 -> scalar ty1 -> result (scalar ty0). (* TODO *)
+Axiom scalar_shr : forall ty0 ty1, scalar ty0 -> scalar ty1 -> result (scalar ty0). (* TODO *)
+
 (** Cast an integer from a [src_ty] to a [tgt_ty] *)
 (* TODO: check the semantics of casts in Rust *)
 Definition scalar_cast (src_ty tgt_ty : scalar_ty) (x : scalar src_ty) : result (scalar tgt_ty) :=
@@ -372,6 +378,76 @@ Definition u32_mul   := @scalar_mul U32.
 Definition u64_mul   := @scalar_mul U64.
 Definition u128_mul  := @scalar_mul U128.
 
+(** Xor *)
+Definition u8_xor := @scalar_xor U8.
+Definition u16_xor := @scalar_xor U16.
+Definition u32_xor := @scalar_xor U32.
+Definition u64_xor := @scalar_xor U64.
+Definition u128_xor := @scalar_xor U128.
+Definition usize_xor := @scalar_xor Usize.
+Definition i8_xor := @scalar_xor I8.
+Definition i16_xor := @scalar_xor I16.
+Definition i32_xor := @scalar_xor I32.
+Definition i64_xor := @scalar_xor I64.
+Definition i128_xor := @scalar_xor I128.
+Definition isize_xor := @scalar_xor Isize.
+
+(** Or *)
+Definition u8_or := @scalar_or U8.
+Definition u16_or := @scalar_or U16.
+Definition u32_or := @scalar_or U32.
+Definition u64_or := @scalar_or U64.
+Definition u128_or := @scalar_or U128.
+Definition usize_or := @scalar_or Usize.
+Definition i8_or := @scalar_or I8.
+Definition i16_or := @scalar_or I16.
+Definition i32_or := @scalar_or I32.
+Definition i64_or := @scalar_or I64.
+Definition i128_or := @scalar_or I128.
+Definition isize_or := @scalar_or Isize.
+
+(** And *)
+Definition u8_and := @scalar_and U8.
+Definition u16_and := @scalar_and U16.
+Definition u32_and := @scalar_and U32.
+Definition u64_and := @scalar_and U64.
+Definition u128_and := @scalar_and U128.
+Definition usize_and := @scalar_and Usize.
+Definition i8_and := @scalar_and I8.
+Definition i16_and := @scalar_and I16.
+Definition i32_and := @scalar_and I32.
+Definition i64_and := @scalar_and I64.
+Definition i128_and := @scalar_and I128.
+Definition isize_and := @scalar_and Isize.
+
+(** Shift left *)
+Definition u8_shl {ty} := @scalar_shl U8 ty.
+Definition u16_shl {ty} := @scalar_shl U16 ty.
+Definition u32_shl {ty} := @scalar_shl U32 ty.
+Definition u64_shl {ty} := @scalar_shl U64 ty.
+Definition u128_shl {ty} := @scalar_shl U128 ty.
+Definition usize_shl {ty} := @scalar_shl Usize ty.
+Definition i8_shl {ty} := @scalar_shl I8 ty.
+Definition i16_shl {ty} := @scalar_shl I16 ty.
+Definition i32_shl {ty} := @scalar_shl I32 ty.
+Definition i64_shl {ty} := @scalar_shl I64 ty.
+Definition i128_shl {ty} := @scalar_shl I128 ty.
+Definition isize_shl {ty} := @scalar_shl Isize ty.
+
+(** Shift right *)
+Definition u8_shr {ty} := @scalar_shr U8 ty.
+Definition u16_shr {ty} := @scalar_shr U16 ty.
+Definition u32_shr {ty} := @scalar_shr U32 ty.
+Definition u64_shr {ty} := @scalar_shr U64 ty.
+Definition u128_shr {ty} := @scalar_shr U128 ty.
+Definition usize_shr {ty} := @scalar_shr Usize ty.
+Definition i8_shr {ty} := @scalar_shr I8 ty.
+Definition i16_shr {ty} := @scalar_shr I16 ty.
+Definition i32_shr {ty} := @scalar_shr I32 ty.
+Definition i64_shr {ty} := @scalar_shr I64 ty.
+Definition i128_shr {ty} := @scalar_shr I128 ty.
+Definition isize_shr {ty} := @scalar_shr Isize ty.
+
 (** Small utility *)
 Definition usize_to_nat (x: usize) : nat := Z.to_nat (to_Z x).
 
-- 
cgit v1.2.3