summaryrefslogtreecommitdiff
path: root/tests/coq/hashmap_on_disk
diff options
context:
space:
mode:
Diffstat (limited to '')
-rw-r--r--tests/coq/hashmap_on_disk/HashmapMain_Funs.v526
-rw-r--r--tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v4
-rw-r--r--tests/coq/hashmap_on_disk/Primitives.v137
3 files changed, 267 insertions, 400 deletions
diff --git a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
index faba0afe..6a7eeb2d 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_Funs.v
@@ -12,69 +12,69 @@ Require Import HashmapMain_FunsExternal.
Include HashmapMain_FunsExternal.
Module HashmapMain_Funs.
-(** [hashmap_main::hashmap::hash_key]: forward function
+(** [hashmap_main::hashmap::hash_key]:
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:
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)
+ (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n1 : usize)
:
result (alloc_vec_Vec (hashmap_List_t T))
:=
match n with
| O => Fail_ OutOfFuel
- | S n1 =>
- if n0 s> 0%usize
+ | S n2 =>
+ if n1 s> 0%usize
then (
- slots0 <- alloc_vec_Vec_push (hashmap_List_t T) slots Hashmap_List_Nil;
- n2 <- usize_sub n0 1%usize;
- hashmap_HashMap_allocate_slots_loop T n1 slots0 n2)
+ v <- alloc_vec_Vec_push (hashmap_List_t T) slots Hashmap_List_Nil;
+ n3 <- usize_sub n1 1%usize;
+ hashmap_HashMap_allocate_slots_loop T n2 v n3)
else Return slots
end
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]: forward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::allocate_slots]:
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)
+ (T : Type) (n : nat) (slots : alloc_vec_Vec (hashmap_List_t T)) (n1 : usize)
:
result (alloc_vec_Vec (hashmap_List_t T))
:=
- hashmap_HashMap_allocate_slots_loop T n slots n0
+ hashmap_HashMap_allocate_slots_loop T n slots n1
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new_with_capacity]: forward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new_with_capacity]:
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) :
result (hashmap_HashMap_t T)
:=
- let v := alloc_vec_Vec_new (hashmap_List_t T) in
- slots <- hashmap_HashMap_allocate_slots T n v capacity;
+ slots <-
+ hashmap_HashMap_allocate_slots T n (alloc_vec_Vec_new (hashmap_List_t T))
+ capacity;
i <- usize_mul capacity max_load_dividend;
- i0 <- usize_div i max_load_divisor;
+ i1 <- usize_div i max_load_divisor;
Return
{|
hashmap_HashMap_num_entries := 0%usize;
hashmap_HashMap_max_load_factor := (max_load_dividend, max_load_divisor);
- hashmap_HashMap_max_load := i0;
+ hashmap_HashMap_max_load := i1;
hashmap_HashMap_slots := slots
|}
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new]: forward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::new]:
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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]: loop 0:
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) :
@@ -82,105 +82,78 @@ Fixpoint hashmap_HashMap_clear_loop
:=
match n with
| O => Fail_ OutOfFuel
- | S n0 =>
- let i0 := alloc_vec_Vec_len (hashmap_List_t T) slots in
- if i s< i0
+ | S n1 =>
+ let i1 := alloc_vec_Vec_len (hashmap_List_t T) slots in
+ if i s< i1
then (
- i1 <- usize_add i 1%usize;
- slots0 <-
- alloc_vec_Vec_index_mut_back (hashmap_List_t T) usize
+ p <-
+ alloc_vec_Vec_index_mut (hashmap_List_t T) usize
(core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T)) slots
- i Hashmap_List_Nil;
- hashmap_HashMap_clear_loop T n0 slots0 i1)
+ i;
+ let (_, index_mut_back) := p in
+ i2 <- usize_add i 1%usize;
+ slots1 <- index_mut_back Hashmap_List_Nil;
+ hashmap_HashMap_clear_loop T n1 slots1 i2)
else Return slots
end
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]: merged forward/backward function
- (there is a single backward function, and the forward function returns ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::clear]:
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)
:=
- v <- hashmap_HashMap_clear_loop T n self.(hashmap_HashMap_slots) 0%usize;
+ back <- hashmap_HashMap_clear_loop T n self.(hashmap_HashMap_slots) 0%usize;
Return
{|
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_HashMap_slots := back
|}
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::len]: forward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::len]:
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:
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
+ result (bool * (hashmap_List_t T))
:=
match n with
| O => Fail_ OutOfFuel
- | S n0 =>
- match ls with
- | Hashmap_List_Cons ckey cvalue tl =>
- if ckey s= key
- then Return false
- else hashmap_HashMap_insert_in_list_loop T n0 key value tl
- | Hashmap_List_Nil => Return true
- end
- end
-.
-
-(** [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
- :=
- 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
- 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)
- :=
- match n with
- | O => Fail_ OutOfFuel
- | S n0 =>
+ | S n1 =>
match ls with
| Hashmap_List_Cons ckey cvalue tl =>
if ckey s= key
- then Return (Hashmap_List_Cons ckey value tl)
+ then Return (false, Hashmap_List_Cons ckey value tl)
else (
- tl0 <- hashmap_HashMap_insert_in_list_loop_back T n0 key value tl;
- Return (Hashmap_List_Cons ckey cvalue tl0))
+ p <- hashmap_HashMap_insert_in_list_loop T n1 key value tl;
+ let (b, back) := p in
+ Return (b, Hashmap_List_Cons ckey cvalue back))
| Hashmap_List_Nil =>
- let l := Hashmap_List_Nil in Return (Hashmap_List_Cons key value l)
+ Return (true, Hashmap_List_Cons key value Hashmap_List_Nil)
end
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]:
Source: 'src/hashmap.rs', lines 97:4-97:71 *)
-Definition hashmap_HashMap_insert_in_list_back
+Definition hashmap_HashMap_insert_in_list
(T : Type) (n : nat) (key : usize) (value : T) (ls : hashmap_List_t T) :
- result (hashmap_List_t T)
+ result (bool * (hashmap_List_t T))
:=
- hashmap_HashMap_insert_in_list_loop_back T n key value ls
+ hashmap_HashMap_insert_in_list_loop T n key value ls
.
-(** [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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert_no_resize]:
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) :
@@ -189,33 +162,27 @@ Definition hashmap_HashMap_insert_no_resize
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 <-
+ p <-
alloc_vec_Vec_index_mut (hashmap_List_t T) usize
(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;
+ let (l, index_mut_back) := p in
+ p1 <- hashmap_HashMap_insert_in_list T n key value l;
+ let (inserted, l1) := p1 in
if inserted
then (
- i0 <- usize_add self.(hashmap_HashMap_num_entries) 1%usize;
- 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_SliceIndexUsizeSliceTInst (hashmap_List_t T))
- self.(hashmap_HashMap_slots) hash_mod l0;
+ i1 <- usize_add self.(hashmap_HashMap_num_entries) 1%usize;
+ v <- index_mut_back l1;
Return
{|
- hashmap_HashMap_num_entries := i0;
+ hashmap_HashMap_num_entries := i1;
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_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_SliceIndexUsizeSliceTInst (hashmap_List_t T))
- self.(hashmap_HashMap_slots) hash_mod l0;
+ v <- index_mut_back l1;
Return
{|
hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
@@ -226,8 +193,7 @@ 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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements_from_list]: loop 0:
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) :
@@ -235,18 +201,17 @@ Fixpoint hashmap_HashMap_move_elements_from_list_loop
:=
match n with
| O => Fail_ OutOfFuel
- | S n0 =>
+ | S n1 =>
match ls with
| 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
+ hm <- hashmap_HashMap_insert_no_resize T n1 ntable k v;
+ hashmap_HashMap_move_elements_from_list_loop T n1 hm tl
| Hashmap_List_Nil => Return ntable
end
end
.
-(** [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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements_from_list]:
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) :
@@ -255,8 +220,7 @@ Definition hashmap_HashMap_move_elements_from_list
hashmap_HashMap_move_elements_from_list_loop T n ntable ls
.
-(** [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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements]: loop 0:
Source: 'src/hashmap.rs', lines 171:4-180:5 *)
Fixpoint hashmap_HashMap_move_elements_loop
(T : Type) (n : nat) (ntable : hashmap_HashMap_t T)
@@ -265,40 +229,39 @@ Fixpoint hashmap_HashMap_move_elements_loop
:=
match n with
| O => Fail_ OutOfFuel
- | S n0 =>
- let i0 := alloc_vec_Vec_len (hashmap_List_t T) slots in
- if i s< i0
+ | S n1 =>
+ let i1 := alloc_vec_Vec_len (hashmap_List_t T) slots in
+ if i s< i1
then (
- l <-
+ p <-
alloc_vec_Vec_index_mut (hashmap_List_t T) usize
(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_SliceIndexUsizeSliceTInst (hashmap_List_t T)) slots
- i l0;
- hashmap_HashMap_move_elements_loop T n0 ntable0 slots0 i1)
+ let (l, index_mut_back) := p in
+ let (ls, l1) := core_mem_replace (hashmap_List_t T) l Hashmap_List_Nil in
+ hm <- hashmap_HashMap_move_elements_from_list T n1 ntable ls;
+ i2 <- usize_add i 1%usize;
+ slots1 <- index_mut_back l1;
+ back_'a <- hashmap_HashMap_move_elements_loop T n1 hm slots1 i2;
+ let (hm1, v) := back_'a in
+ Return (hm1, v))
else Return (ntable, slots)
end
.
-(** [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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::move_elements]:
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) :
result ((hashmap_HashMap_t T) * (alloc_vec_Vec (hashmap_List_t T)))
:=
- hashmap_HashMap_move_elements_loop T n ntable slots i
+ back_'a <- hashmap_HashMap_move_elements_loop T n ntable slots i;
+ let (hm, v) := back_'a in
+ Return (hm, v)
.
-(** [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 ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::try_resize]:
Source: 'src/hashmap.rs', lines 140:4-140:28 *)
Definition hashmap_HashMap_try_resize
(T : Type) (n : nat) (self : hashmap_HashMap_t T) :
@@ -308,72 +271,71 @@ Definition hashmap_HashMap_try_resize
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_HashMap_max_load_factor) in
- i1 <- usize_div n1 i;
- if capacity s<= i1
+ let (i, i1) := self.(hashmap_HashMap_max_load_factor) in
+ i2 <- usize_div n1 i;
+ if capacity s<= i2
then (
- i2 <- usize_mul capacity 2%usize;
- ntable <- hashmap_HashMap_new_with_capacity T n i2 i i0;
+ i3 <- usize_mul capacity 2%usize;
+ ntable <- hashmap_HashMap_new_with_capacity T n i3 i i1;
p <-
hashmap_HashMap_move_elements T n ntable self.(hashmap_HashMap_slots)
0%usize;
- let (ntable0, _) := p in
+ let (ntable1, _) := p in
Return
{|
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)
+ hashmap_HashMap_max_load_factor := (i, i1);
+ hashmap_HashMap_max_load := ntable1.(hashmap_HashMap_max_load);
+ hashmap_HashMap_slots := ntable1.(hashmap_HashMap_slots)
|})
else
Return
{|
hashmap_HashMap_num_entries := self.(hashmap_HashMap_num_entries);
- hashmap_HashMap_max_load_factor := (i, i0);
+ hashmap_HashMap_max_load_factor := (i, i1);
hashmap_HashMap_max_load := self.(hashmap_HashMap_max_load);
hashmap_HashMap_slots := self.(hashmap_HashMap_slots)
|}
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert]: merged forward/backward function
- (there is a single backward function, and the forward function returns ())
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::insert]:
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)
:=
- 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
+ hm <- hashmap_HashMap_insert_no_resize T n self key value;
+ i <- hashmap_HashMap_len T hm;
+ if i s> hm.(hashmap_HashMap_max_load)
+ then hashmap_HashMap_try_resize T n hm
+ else Return hm
.
-(** [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:
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
| O => Fail_ OutOfFuel
- | S n0 =>
+ | S n1 =>
match ls with
- | Hashmap_List_Cons ckey t tl =>
+ | Hashmap_List_Cons ckey _ tl =>
if ckey s= key
then Return true
- else hashmap_HashMap_contains_key_in_list_loop T n0 key tl
+ else hashmap_HashMap_contains_key_in_list_loop T n1 key tl
| Hashmap_List_Nil => Return false
end
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]:
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]:
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) :
@@ -389,31 +351,31 @@ 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:
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
| O => Fail_ OutOfFuel
- | S n0 =>
+ | S n1 =>
match ls with
| Hashmap_List_Cons ckey cvalue tl =>
if ckey s= key
then Return cvalue
- else hashmap_HashMap_get_in_list_loop T n0 key tl
+ else hashmap_HashMap_get_in_list_loop T n1 key tl
| Hashmap_List_Nil => Fail_ Failure
end
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]:
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]:
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 :=
@@ -427,292 +389,208 @@ 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:
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
- | O => Fail_ OutOfFuel
- | S n0 =>
- match ls with
- | Hashmap_List_Cons ckey cvalue tl =>
- if ckey s= key
- then Return cvalue
- else hashmap_HashMap_get_mut_in_list_loop T n0 tl key
- | Hashmap_List_Nil => Fail_ Failure
- end
- end
-.
-
-(** [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
- 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)
+ (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) :
+ result (T * (T -> result (hashmap_List_t T)))
:=
match n with
| O => Fail_ OutOfFuel
- | S n0 =>
+ | S n1 =>
match ls with
| Hashmap_List_Cons ckey cvalue tl =>
if ckey s= key
- then Return (Hashmap_List_Cons ckey ret tl)
+ then
+ let back_'a := fun (ret : T) => Return (Hashmap_List_Cons ckey ret tl)
+ in
+ Return (cvalue, back_'a)
else (
- tl0 <- hashmap_HashMap_get_mut_in_list_loop_back T n0 tl key ret;
- Return (Hashmap_List_Cons ckey cvalue tl0))
+ p <- hashmap_HashMap_get_mut_in_list_loop T n1 tl key;
+ let (t, back_'a) := p in
+ let back_'a1 :=
+ fun (ret : T) =>
+ tl1 <- back_'a ret; Return (Hashmap_List_Cons ckey cvalue tl1) in
+ Return (t, back_'a1))
| Hashmap_List_Nil => Fail_ Failure
end
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]:
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)
+Definition hashmap_HashMap_get_mut_in_list
+ (T : Type) (n : nat) (ls : hashmap_List_t T) (key : usize) :
+ result (T * (T -> result (hashmap_List_t T)))
:=
- hashmap_HashMap_get_mut_in_list_loop_back T n ls key ret
+ p <- hashmap_HashMap_get_mut_in_list_loop T n ls key;
+ let (t, back_'a) := p in
+ Return (t, back_'a)
.
-(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]: forward function
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::get_mut]:
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;
- let i := alloc_vec_Vec_len (hashmap_List_t T) self.(hashmap_HashMap_slots) in
- hash_mod <- usize_rem hash i;
- l <-
- alloc_vec_Vec_index_mut (hashmap_List_t T) usize
- (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_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)
+ (T : Type) (n : nat) (self : hashmap_HashMap_t T) (key : usize) :
+ result (T * (T -> result (hashmap_HashMap_t 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 <-
+ p <-
alloc_vec_Vec_index_mut (hashmap_List_t T) usize
(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_SliceIndexUsizeSliceTInst (hashmap_List_t T))
- self.(hashmap_HashMap_slots) hash_mod l0;
- Return
- {|
- 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_main::hashmap::HashMap<T>}::remove_from_list]: loop 0: forward function
+ let (l, index_mut_back) := p in
+ p1 <- hashmap_HashMap_get_mut_in_list T n l key;
+ let (t, get_mut_in_list_back) := p1 in
+ let back_'a :=
+ fun (ret : T) =>
+ l1 <- get_mut_in_list_back ret;
+ v <- index_mut_back l1;
+ Return
+ {|
+ 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
+ |} in
+ Return (t, back_'a)
+.
+
+(** [hashmap_main::hashmap::{hashmap_main::hashmap::HashMap<T>}::remove_from_list]: loop 0:
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)
+ result ((option T) * (hashmap_List_t T))
:=
match n with
| O => Fail_ OutOfFuel
- | S n0 =>
+ | S n1 =>
match ls with
| Hashmap_List_Cons ckey t tl =>
if ckey s= key
then
- let mv_ls :=
+ let (mv_ls, _) :=
core_mem_replace (hashmap_List_t T) (Hashmap_List_Cons ckey t tl)
Hashmap_List_Nil in
match mv_ls with
- | Hashmap_List_Cons i cvalue tl0 => Return (Some cvalue)
+ | Hashmap_List_Cons _ cvalue tl1 => Return (Some cvalue, tl1)
| Hashmap_List_Nil => Fail_ Failure
end
- else hashmap_HashMap_remove_from_list_loop T n0 key tl
- | Hashmap_List_Nil => Return None
+ else (
+ p <- hashmap_HashMap_remove_from_list_loop T n1 key tl;
+ let (o, back) := p in
+ Return (o, Hashmap_List_Cons ckey t back))
+ | Hashmap_List_Nil => Return (None, Hashmap_List_Nil)
end
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]:
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)
+ result ((option T) * (hashmap_List_t T))
:=
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
- 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)
- :=
- match n with
- | O => Fail_ OutOfFuel
- | S n0 =>
- match ls with
- | Hashmap_List_Cons ckey t tl =>
- if ckey s= key
- then
- let mv_ls :=
- core_mem_replace (hashmap_List_t T) (Hashmap_List_Cons ckey t tl)
- Hashmap_List_Nil in
- match mv_ls with
- | Hashmap_List_Cons i cvalue tl0 => Return tl0
- | Hashmap_List_Nil => Fail_ Failure
- end
- else (
- 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_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)
- :=
- 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]:
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)
+ result ((option T) * (hashmap_HashMap_t 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 <-
+ p <-
alloc_vec_Vec_index_mut (hashmap_List_t T) usize
(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
- | None => Return None
- | Some x0 =>
- _ <- usize_sub self.(hashmap_HashMap_num_entries) 1%usize; Return (Some x0)
- end
-.
-
-(** [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)
- :=
- 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 <-
- alloc_vec_Vec_index_mut (hashmap_List_t T) usize
- (core_slice_index_SliceIndexUsizeSliceTInst (hashmap_List_t T))
- self.(hashmap_HashMap_slots) hash_mod;
- x <- hashmap_HashMap_remove_from_list T n key l;
+ let (l, index_mut_back) := p in
+ p1 <- hashmap_HashMap_remove_from_list T n key l;
+ let (x, l1) := p1 in
match x with
| None =>
- 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_SliceIndexUsizeSliceTInst (hashmap_List_t T))
- self.(hashmap_HashMap_slots) hash_mod l0;
- Return
+ v <- index_mut_back l1;
+ Return (None,
{|
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_HashMap_num_entries) 1%usize;
- 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_SliceIndexUsizeSliceTInst (hashmap_List_t T))
- self.(hashmap_HashMap_slots) hash_mod l0;
- Return
+ |})
+ | Some x1 =>
+ i1 <- usize_sub self.(hashmap_HashMap_num_entries) 1%usize;
+ v <- index_mut_back l1;
+ Return (Some x1,
{|
- hashmap_HashMap_num_entries := i0;
+ hashmap_HashMap_num_entries := i1;
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
+(** [hashmap_main::hashmap::test1]:
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;
- 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;
+ hm1 <- hashmap_HashMap_insert u64 n hm 0%usize 42%u64;
+ hm2 <- hashmap_HashMap_insert u64 n hm1 128%usize 18%u64;
+ hm3 <- hashmap_HashMap_insert u64 n hm2 1024%usize 138%u64;
+ hm4 <- hashmap_HashMap_insert u64 n hm3 1056%usize 256%u64;
+ i <- hashmap_HashMap_get u64 n hm4 128%usize;
if negb (i s= 18%u64)
then Fail_ Failure
else (
- 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)
+ p <- hashmap_HashMap_get_mut u64 n hm4 1024%usize;
+ let (_, get_mut_back) := p in
+ hm5 <- get_mut_back 56%u64;
+ i1 <- hashmap_HashMap_get u64 n hm5 1024%usize;
+ if negb (i1 s= 56%u64)
then Fail_ Failure
else (
- x <- hashmap_HashMap_remove u64 n hm4 1024%usize;
+ p1 <- hashmap_HashMap_remove u64 n hm5 1024%usize;
+ let (x, hm6) := p1 in
match x with
| None => Fail_ Failure
- | Some x0 =>
- if negb (x0 s= 56%u64)
+ | Some x1 =>
+ if negb (x1 s= 56%u64)
then Fail_ Failure
else (
- 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)
+ i2 <- hashmap_HashMap_get u64 n hm6 0%usize;
+ if negb (i2 s= 42%u64)
then Fail_ Failure
else (
- i2 <- hashmap_HashMap_get u64 n hm5 128%usize;
- if negb (i2 s= 18%u64)
+ i3 <- hashmap_HashMap_get u64 n hm6 128%usize;
+ if negb (i3 s= 18%u64)
then Fail_ Failure
else (
- i3 <- hashmap_HashMap_get u64 n hm5 1056%usize;
- if negb (i3 s= 256%u64) then Fail_ Failure else Return tt)))
+ i4 <- hashmap_HashMap_get u64 n hm6 1056%usize;
+ if negb (i4 s= 256%u64) then Fail_ Failure else Return tt)))
end))
.
-(** [hashmap_main::insert_on_disk]: forward function
+(** [hashmap_main::insert_on_disk]:
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;
- let (st0, hm) := p in
- hm0 <- hashmap_HashMap_insert u64 n hm key value;
- p0 <- hashmap_utils_serialize hm0 st0;
- let (st1, _) := p0 in
- Return (st1, tt)
+ let (st1, hm) := p in
+ hm1 <- hashmap_HashMap_insert u64 n hm key value;
+ p1 <- hashmap_utils_serialize hm1 st1;
+ let (st2, _) := p1 in
+ Return (st2, tt)
.
-(** [hashmap_main::main]: forward function
+(** [hashmap_main::main]:
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_FunsExternal_Template.v b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
index e10d02f6..fb2e052a 100644
--- a/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
+++ b/tests/coq/hashmap_on_disk/HashmapMain_FunsExternal_Template.v
@@ -11,13 +11,13 @@ Require Import HashmapMain_Types.
Include HashmapMain_Types.
Module HashmapMain_FunsExternal_Template.
-(** [hashmap_main::hashmap_utils::deserialize]: forward function
+(** [hashmap_main::hashmap_utils::deserialize]:
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]:
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/Primitives.v b/tests/coq/hashmap_on_disk/Primitives.v
index 84280b96..990e27e4 100644
--- a/tests/coq/hashmap_on_disk/Primitives.v
+++ b/tests/coq/hashmap_on_disk/Primitives.v
@@ -67,8 +67,7 @@ Definition string := Coq.Strings.String.string.
Definition char := Coq.Strings.Ascii.ascii.
Definition char_of_byte := Coq.Strings.Ascii.ascii_of_byte.
-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 .
+Definition core_mem_replace (a : Type) (x : a) (y : a) : a * a := (x, x) .
Record mut_raw_ptr (T : Type) := { mut_raw_ptr_v : T }.
Record const_raw_ptr (T : Type) := { const_raw_ptr_v : T }.
@@ -504,13 +503,15 @@ 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;
+ core_ops_index_IndexMut_index_mut :
+ Self ->
+ Idx ->
+ result (core_ops_index_IndexMut_indexInst.(core_ops_index_Index_Output) *
+ (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 {
@@ -524,13 +525,14 @@ 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;
+ core_ops_deref_DerefMut_deref_mut :
+ Self ->
+ result (core_ops_deref_DerefMut_derefInst.(core_ops_deref_Deref_target) *
+ (core_ops_deref_DerefMut_derefInst.(core_ops_deref_Deref_target) -> result Self));
}.
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;
@@ -543,8 +545,8 @@ 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.
+Definition alloc_boxed_Box_deref_mut (T : Type) (x : T) : result (T * (T -> result T)) :=
+ Return (x, fun x => Return x).
(* Trait instance *)
Definition alloc_boxed_Box_coreopsDerefInst (Self : Type) : core_ops_deref_Deref Self := {|
@@ -556,7 +558,6 @@ Definition alloc_boxed_Box_coreopsDerefInst (Self : Type) : core_ops_deref_Deref
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;
|}.
@@ -584,6 +585,13 @@ 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).
+Definition array_index_mut_usize (T : Type) (n : usize) (a : array T n) (i : usize) :
+ result (T * (T -> result (array T n))) :=
+ match array_index_usize T n a i with
+ | Fail_ e => Fail_ e
+ | Return x => Return (x, array_update_usize T n a i)
+ end.
+
(*** Slice *)
Definition slice T := { l: list T | Z.of_nat (length l) <= usize_max}.
@@ -591,11 +599,25 @@ Axiom slice_len : forall (T : Type) (s : slice T), usize.
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).
+Definition slice_index_mut_usize (T : Type) (s : slice T) (i : usize) :
+ result (T * (T -> result (slice T))) :=
+ match slice_index_usize T s i with
+ | Fail_ e => Fail_ e
+ | Return x => Return (x, slice_update_usize T s i)
+ end.
+
(*** Subslices *)
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).
+Definition array_to_slice_mut (T : Type) (n : usize) (a : array T n) :
+ result (slice T * (slice T -> result (array T n))) :=
+ match array_to_slice T n a with
+ | Fail_ e => Fail_ e
+ | Return x => Return (x, array_from_slice T n a)
+ end.
+
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).
@@ -639,16 +661,9 @@ Definition alloc_vec_Vec_bind {A B} (v: alloc_vec_Vec A) (f: list A -> result (l
| right _ => Fail_ Failure
end.
-(* The **forward** function shouldn't be used *)
-Definition alloc_vec_Vec_push_fwd (T: Type) (v: alloc_vec_Vec T) (x: T) : unit := tt.
-
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 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 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)
@@ -661,6 +676,14 @@ Axiom alloc_vec_Vec_index_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : u
(* Helper *)
Axiom alloc_vec_Vec_update_usize : forall {T : Type} (v : alloc_vec_Vec T) (i : usize) (x : T), result (alloc_vec_Vec T).
+Definition alloc_vec_Vec_index_mut_usize {T : Type} (v: alloc_vec_Vec T) (i: usize) :
+ result (T * (T -> result (alloc_vec_Vec T))) :=
+ match alloc_vec_Vec_index_usize v i with
+ | Return x =>
+ Return (x, alloc_vec_Vec_update_usize v i)
+ | Fail_ e => Fail_ e
+ end.
+
(* Trait declaration: [core::slice::index::private_slice_index::Sealed] *)
Definition core_slice_index_private_slice_index_Sealed (self : Type) := unit.
@@ -669,25 +692,23 @@ Record core_slice_index_SliceIndex (Self T : Type) := mk_core_slice_index_SliceI
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_mut :
+ Self -> T -> result (option core_slice_index_SliceIndex_Output * (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;
+ core_slice_index_SliceIndex_index_mut :
+ Self -> T -> result (core_slice_index_SliceIndex_Output * (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
@@ -704,11 +725,9 @@ Axiom core_slice_index_RangeUsize_get : forall (T : Type) (i : core_ops_range_Ra
(* [core::slice::index::Range::get_mut]: forward function *)
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_RangeUsize_get_mut_back :
- forall (T : Type), core_ops_range_Range usize -> slice T -> option (slice T) -> result (slice T).
+ forall (T : Type),
+ core_ops_range_Range usize -> slice T ->
+ result (option (slice T) * (option (slice T) -> result (slice T))).
(* [core::slice::index::Range::get_unchecked]: forward function *)
Definition core_slice_index_RangeUsize_get_unchecked
@@ -732,21 +751,14 @@ Axiom core_slice_index_RangeUsize_index :
(* [core::slice::index::Range::index_mut]: forward function *)
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_RangeUsize_index_mut_back :
- forall (T : Type), core_ops_range_Range usize -> slice T -> slice T -> result (slice T).
+ forall (T : Type), core_ops_range_Range usize -> slice T -> result (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).
+ slice T -> Idx ->
+ result (inst.(core_slice_index_SliceIndex_Output) *
+ (inst.(core_slice_index_SliceIndex_Output) -> result (slice T))).
(* [core::array::[T; N]::index]: forward function *)
Axiom core_array_Array_index :
@@ -756,12 +768,9 @@ Axiom core_array_Array_index :
(* [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).
+ (a : array T N) (i : Idx),
+ result (inst.(core_ops_index_IndexMut_indexInst).(core_ops_index_Index_Output) *
+ (inst.(core_ops_index_IndexMut_indexInst).(core_ops_index_Index_Output) -> result (array T N))).
(* Trait implementation: [core::slice::index::private_slice_index::Range] *)
Definition core_slice_index_private_slice_index_SealedRangeUsizeInst
@@ -774,12 +783,10 @@ Definition core_slice_index_SliceIndexRangeUsizeSliceTInst (T : Type) :
core_slice_index_SliceIndex_Output := slice 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]] *)
@@ -796,7 +803,6 @@ Definition core_ops_index_IndexMutSliceTIInst (T Idx : Type)
core_ops_index_IndexMut (slice T) Idx := {|
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]] *)
@@ -813,18 +819,14 @@ Definition core_ops_index_IndexMutArrayInst (T Idx : Type) (N : usize)
core_ops_index_IndexMut (array T N) Idx := {|
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;
|}.
(* [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).
+Axiom core_slice_index_usize_get_mut :
+ forall (T : Type), usize -> slice T -> result (option T * (option T -> result (slice T))).
(* [core::slice::index::usize::get_unchecked]: forward function *)
Axiom core_slice_index_usize_get_unchecked :
@@ -838,11 +840,8 @@ Axiom core_slice_index_usize_get_unchecked_mut :
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).
+Axiom core_slice_index_usize_index_mut :
+ forall (T : Type), usize -> slice T -> result (T * (T -> result (slice T))).
(* Trait implementation: [core::slice::index::private_slice_index::usize] *)
Definition core_slice_index_private_slice_index_SealedUsizeInst
@@ -855,12 +854,10 @@ Definition core_slice_index_SliceIndexUsizeSliceTInst (T : Type) :
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 *)
@@ -869,12 +866,9 @@ Axiom alloc_vec_Vec_index : forall (T Idx : Type) (inst : core_slice_index_Slice
(* [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).
+ (Self : alloc_vec_Vec T) (i : Idx),
+ result (inst.(core_slice_index_SliceIndex_Output) *
+ (inst.(core_slice_index_SliceIndex_Output) -> result (alloc_vec_Vec T))).
(* Trait implementation: [alloc::vec::Vec] *)
Definition alloc_vec_Vec_coreopsindexIndexInst (T Idx : Type)
@@ -890,7 +884,6 @@ Definition alloc_vec_Vec_coreopsindexIndexMutInst (T Idx : Type)
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 *)
@@ -901,10 +894,6 @@ Axiom alloc_vec_Vec_index_eq : forall {a : Type} (v : alloc_vec_Vec a) (i : usiz
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_SliceIndexUsizeSliceTInst a) v i x =
- alloc_vec_Vec_update_usize v i x.
+ alloc_vec_Vec_index_mut_usize v i.
End Primitives.