From 37e8a0f5ff7d964eb9525fef765b38e44f79302b Mon Sep 17 00:00:00 2001 From: Nadrieril Date: Fri, 24 May 2024 15:48:27 +0200 Subject: Update test outputs --- tests/coq/misc/Bitwise.v | 10 ++-- tests/coq/misc/Constants.v | 62 +++++++++---------- tests/coq/misc/External_Funs.v | 4 +- tests/coq/misc/Loops.v | 98 +++++++++++++++--------------- tests/coq/misc/NoNestedBorrows.v | 126 +++++++++++++++++++-------------------- tests/coq/misc/Paper.v | 18 +++--- tests/coq/misc/PoloniusList.v | 4 +- 7 files changed, 161 insertions(+), 161 deletions(-) (limited to 'tests/coq/misc') diff --git a/tests/coq/misc/Bitwise.v b/tests/coq/misc/Bitwise.v index 539141e5..d0dbfd51 100644 --- a/tests/coq/misc/Bitwise.v +++ b/tests/coq/misc/Bitwise.v @@ -9,29 +9,29 @@ Local Open Scope Primitives_scope. Module Bitwise. (** [bitwise::shift_u32]: - Source: 'tests/src/bitwise.rs', lines 3:0-3:31 *) + Source: 'tests/src/bitwise.rs', lines 4:0-4:31 *) Definition shift_u32 (a : u32) : result u32 := t <- u32_shr a 16%usize; u32_shl t 16%usize . (** [bitwise::shift_i32]: - Source: 'tests/src/bitwise.rs', lines 10:0-10:31 *) + Source: 'tests/src/bitwise.rs', lines 11:0-11:31 *) Definition shift_i32 (a : i32) : result i32 := t <- i32_shr a 16%isize; i32_shl t 16%isize . (** [bitwise::xor_u32]: - Source: 'tests/src/bitwise.rs', lines 17:0-17:37 *) + Source: 'tests/src/bitwise.rs', lines 18:0-18:37 *) Definition xor_u32 (a : u32) (b : u32) : result u32 := Ok (u32_xor a b). (** [bitwise::or_u32]: - Source: 'tests/src/bitwise.rs', lines 21:0-21:36 *) + Source: 'tests/src/bitwise.rs', lines 22:0-22:36 *) Definition or_u32 (a : u32) (b : u32) : result u32 := Ok (u32_or a b). (** [bitwise::and_u32]: - Source: 'tests/src/bitwise.rs', lines 25:0-25:37 *) + Source: 'tests/src/bitwise.rs', lines 26:0-26:37 *) Definition and_u32 (a : u32) (b : u32) : result u32 := Ok (u32_and a b). diff --git a/tests/coq/misc/Constants.v b/tests/coq/misc/Constants.v index a5aba663..c3ecdb83 100644 --- a/tests/coq/misc/Constants.v +++ b/tests/coq/misc/Constants.v @@ -9,37 +9,37 @@ Local Open Scope Primitives_scope. Module Constants. (** [constants::X0] - Source: 'tests/src/constants.rs', lines 5:0-5:17 *) + Source: 'tests/src/constants.rs', lines 7:0-7:17 *) Definition x0_body : result u32 := Ok 0%u32. Definition x0 : u32 := x0_body%global. (** [constants::X1] - Source: 'tests/src/constants.rs', lines 7:0-7:17 *) + Source: 'tests/src/constants.rs', lines 9:0-9:17 *) Definition x1_body : result u32 := Ok core_u32_max. Definition x1 : u32 := x1_body%global. (** [constants::X2] - Source: 'tests/src/constants.rs', lines 10:0-10:17 *) + Source: 'tests/src/constants.rs', lines 12:0-12:17 *) Definition x2_body : result u32 := Ok 3%u32. Definition x2 : u32 := x2_body%global. (** [constants::incr]: - Source: 'tests/src/constants.rs', lines 17:0-17:32 *) + Source: 'tests/src/constants.rs', lines 19:0-19:32 *) Definition incr (n : u32) : result u32 := u32_add n 1%u32. (** [constants::X3] - Source: 'tests/src/constants.rs', lines 15:0-15:17 *) + Source: 'tests/src/constants.rs', lines 17:0-17:17 *) Definition x3_body : result u32 := incr 32%u32. Definition x3 : u32 := x3_body%global. (** [constants::mk_pair0]: - Source: 'tests/src/constants.rs', lines 23:0-23:51 *) + Source: 'tests/src/constants.rs', lines 25:0-25:51 *) Definition mk_pair0 (x : u32) (y1 : u32) : result (u32 * u32) := Ok (x, y1). (** [constants::Pair] - Source: 'tests/src/constants.rs', lines 36:0-36:23 *) + Source: 'tests/src/constants.rs', lines 38:0-38:23 *) Record Pair_t (T1 T2 : Type) := mkPair_t { pair_x : T1; pair_y : T2; }. Arguments mkPair_t { _ _ }. @@ -47,130 +47,130 @@ Arguments pair_x { _ _ }. Arguments pair_y { _ _ }. (** [constants::mk_pair1]: - Source: 'tests/src/constants.rs', lines 27:0-27:55 *) + Source: 'tests/src/constants.rs', lines 29:0-29:55 *) Definition mk_pair1 (x : u32) (y1 : u32) : result (Pair_t u32 u32) := Ok {| pair_x := x; pair_y := y1 |} . (** [constants::P0] - Source: 'tests/src/constants.rs', lines 31:0-31:24 *) + Source: 'tests/src/constants.rs', lines 33:0-33:24 *) Definition p0_body : result (u32 * u32) := mk_pair0 0%u32 1%u32. Definition p0 : (u32 * u32) := p0_body%global. (** [constants::P1] - Source: 'tests/src/constants.rs', lines 32:0-32:28 *) + Source: 'tests/src/constants.rs', lines 34:0-34:28 *) Definition p1_body : result (Pair_t u32 u32) := mk_pair1 0%u32 1%u32. Definition p1 : Pair_t u32 u32 := p1_body%global. (** [constants::P2] - Source: 'tests/src/constants.rs', lines 33:0-33:24 *) + Source: 'tests/src/constants.rs', lines 35:0-35:24 *) Definition p2_body : result (u32 * u32) := Ok (0%u32, 1%u32). Definition p2 : (u32 * u32) := p2_body%global. (** [constants::P3] - Source: 'tests/src/constants.rs', lines 34:0-34:28 *) + Source: 'tests/src/constants.rs', lines 36:0-36:28 *) Definition p3_body : result (Pair_t u32 u32) := Ok {| pair_x := 0%u32; pair_y := 1%u32 |} . Definition p3 : Pair_t u32 u32 := p3_body%global. (** [constants::Wrap] - Source: 'tests/src/constants.rs', lines 49:0-49:18 *) + Source: 'tests/src/constants.rs', lines 51:0-51:18 *) Record Wrap_t (T : Type) := mkWrap_t { wrap_value : T; }. Arguments mkWrap_t { _ }. Arguments wrap_value { _ }. (** [constants::{constants::Wrap}::new]: - Source: 'tests/src/constants.rs', lines 54:4-54:41 *) + Source: 'tests/src/constants.rs', lines 56:4-56:41 *) Definition wrap_new (T : Type) (value : T) : result (Wrap_t T) := Ok {| wrap_value := value |} . (** [constants::Y] - Source: 'tests/src/constants.rs', lines 41:0-41:22 *) + Source: 'tests/src/constants.rs', lines 43:0-43:22 *) Definition y_body : result (Wrap_t i32) := wrap_new i32 2%i32. Definition y : Wrap_t i32 := y_body%global. (** [constants::unwrap_y]: - Source: 'tests/src/constants.rs', lines 43:0-43:30 *) + Source: 'tests/src/constants.rs', lines 45:0-45:30 *) Definition unwrap_y : result i32 := Ok y.(wrap_value). (** [constants::YVAL] - Source: 'tests/src/constants.rs', lines 47:0-47:19 *) + Source: 'tests/src/constants.rs', lines 49:0-49:19 *) Definition yval_body : result i32 := unwrap_y. Definition yval : i32 := yval_body%global. (** [constants::get_z1::Z1] - Source: 'tests/src/constants.rs', lines 62:4-62:17 *) + Source: 'tests/src/constants.rs', lines 64:4-64:17 *) Definition get_z1_z1_body : result i32 := Ok 3%i32. Definition get_z1_z1 : i32 := get_z1_z1_body%global. (** [constants::get_z1]: - Source: 'tests/src/constants.rs', lines 61:0-61:28 *) + Source: 'tests/src/constants.rs', lines 63:0-63:28 *) Definition get_z1 : result i32 := Ok get_z1_z1. (** [constants::add]: - Source: 'tests/src/constants.rs', lines 66:0-66:39 *) + Source: 'tests/src/constants.rs', lines 68:0-68:39 *) Definition add (a : i32) (b : i32) : result i32 := i32_add a b. (** [constants::Q1] - Source: 'tests/src/constants.rs', lines 74:0-74:17 *) + Source: 'tests/src/constants.rs', lines 76:0-76:17 *) Definition q1_body : result i32 := Ok 5%i32. Definition q1 : i32 := q1_body%global. (** [constants::Q2] - Source: 'tests/src/constants.rs', lines 75:0-75:17 *) + Source: 'tests/src/constants.rs', lines 77:0-77:17 *) Definition q2_body : result i32 := Ok q1. Definition q2 : i32 := q2_body%global. (** [constants::Q3] - Source: 'tests/src/constants.rs', lines 76:0-76:17 *) + Source: 'tests/src/constants.rs', lines 78:0-78:17 *) Definition q3_body : result i32 := add q2 3%i32. Definition q3 : i32 := q3_body%global. (** [constants::get_z2]: - Source: 'tests/src/constants.rs', lines 70:0-70:28 *) + Source: 'tests/src/constants.rs', lines 72:0-72:28 *) Definition get_z2 : result i32 := i <- get_z1; i1 <- add i q3; add q1 i1. (** [constants::S1] - Source: 'tests/src/constants.rs', lines 80:0-80:18 *) + Source: 'tests/src/constants.rs', lines 82:0-82:18 *) Definition s1_body : result u32 := Ok 6%u32. Definition s1 : u32 := s1_body%global. (** [constants::S2] - Source: 'tests/src/constants.rs', lines 81:0-81:18 *) + Source: 'tests/src/constants.rs', lines 83:0-83:18 *) Definition s2_body : result u32 := incr s1. Definition s2 : u32 := s2_body%global. (** [constants::S3] - Source: 'tests/src/constants.rs', lines 82:0-82:29 *) + Source: 'tests/src/constants.rs', lines 84:0-84:29 *) Definition s3_body : result (Pair_t u32 u32) := Ok p3. Definition s3 : Pair_t u32 u32 := s3_body%global. (** [constants::S4] - Source: 'tests/src/constants.rs', lines 83:0-83:29 *) + Source: 'tests/src/constants.rs', lines 85:0-85:29 *) Definition s4_body : result (Pair_t u32 u32) := mk_pair1 7%u32 8%u32. Definition s4 : Pair_t u32 u32 := s4_body%global. (** [constants::V] - Source: 'tests/src/constants.rs', lines 86:0-86:31 *) + Source: 'tests/src/constants.rs', lines 88:0-88:31 *) Record V_t (T : Type) (N : usize) := mkV_t { v_x : array T N; }. Arguments mkV_t { _ _ }. Arguments v_x { _ _ }. (** [constants::{constants::V#1}::LEN] - Source: 'tests/src/constants.rs', lines 91:4-91:24 *) + Source: 'tests/src/constants.rs', lines 93:4-93:24 *) Definition v_len_body (T : Type) (N : usize) : result usize := Ok N. Definition v_len (T : Type) (N : usize) : usize := (v_len_body T N)%global. (** [constants::use_v]: - Source: 'tests/src/constants.rs', lines 94:0-94:42 *) + Source: 'tests/src/constants.rs', lines 96:0-96:42 *) Definition use_v (T : Type) (N : usize) : result usize := Ok (v_len T N). diff --git a/tests/coq/misc/External_Funs.v b/tests/coq/misc/External_Funs.v index d0de80d9..18586012 100644 --- a/tests/coq/misc/External_Funs.v +++ b/tests/coq/misc/External_Funs.v @@ -20,14 +20,14 @@ Definition core_marker_CopyU32 : core_marker_Copy_t u32 := {| |}. (** [external::use_get]: - Source: 'tests/src/external.rs', lines 5:0-5:37 *) + Source: 'tests/src/external.rs', lines 8:0-8:37 *) Definition use_get (rc : core_cell_Cell_t u32) (st : state) : result (state * u32) := core_cell_Cell_get u32 core_marker_CopyU32 rc st . (** [external::incr]: - Source: 'tests/src/external.rs', lines 9:0-9:31 *) + Source: 'tests/src/external.rs', lines 12:0-12:31 *) Definition incr (rc : core_cell_Cell_t u32) (st : state) : result (state * (core_cell_Cell_t u32)) diff --git a/tests/coq/misc/Loops.v b/tests/coq/misc/Loops.v index bf0a8bc1..bc8708f4 100644 --- a/tests/coq/misc/Loops.v +++ b/tests/coq/misc/Loops.v @@ -9,7 +9,7 @@ Local Open Scope Primitives_scope. Module Loops. (** [loops::sum]: loop 0: - Source: 'tests/src/loops.rs', lines 4:0-14:1 *) + Source: 'tests/src/loops.rs', lines 7:0-17:1 *) Fixpoint sum_loop (n : nat) (max : u32) (i : u32) (s : u32) : result u32 := match n with | O => Fail_ OutOfFuel @@ -21,13 +21,13 @@ Fixpoint sum_loop (n : nat) (max : u32) (i : u32) (s : u32) : result u32 := . (** [loops::sum]: - Source: 'tests/src/loops.rs', lines 4:0-4:27 *) + Source: 'tests/src/loops.rs', lines 7:0-7:27 *) Definition sum (n : nat) (max : u32) : result u32 := sum_loop n max 0%u32 0%u32 . (** [loops::sum_with_mut_borrows]: loop 0: - Source: 'tests/src/loops.rs', lines 19:0-31:1 *) + Source: 'tests/src/loops.rs', lines 22:0-34:1 *) Fixpoint sum_with_mut_borrows_loop (n : nat) (max : u32) (i : u32) (s : u32) : result u32 := match n with @@ -43,13 +43,13 @@ Fixpoint sum_with_mut_borrows_loop . (** [loops::sum_with_mut_borrows]: - Source: 'tests/src/loops.rs', lines 19:0-19:44 *) + Source: 'tests/src/loops.rs', lines 22:0-22:44 *) Definition sum_with_mut_borrows (n : nat) (max : u32) : result u32 := sum_with_mut_borrows_loop n max 0%u32 0%u32 . (** [loops::sum_with_shared_borrows]: loop 0: - Source: 'tests/src/loops.rs', lines 34:0-48:1 *) + Source: 'tests/src/loops.rs', lines 37:0-51:1 *) Fixpoint sum_with_shared_borrows_loop (n : nat) (max : u32) (i : u32) (s : u32) : result u32 := match n with @@ -65,13 +65,13 @@ Fixpoint sum_with_shared_borrows_loop . (** [loops::sum_with_shared_borrows]: - Source: 'tests/src/loops.rs', lines 34:0-34:47 *) + Source: 'tests/src/loops.rs', lines 37:0-37:47 *) Definition sum_with_shared_borrows (n : nat) (max : u32) : result u32 := sum_with_shared_borrows_loop n max 0%u32 0%u32 . (** [loops::sum_array]: loop 0: - Source: 'tests/src/loops.rs', lines 50:0-58:1 *) + Source: 'tests/src/loops.rs', lines 53:0-61:1 *) Fixpoint sum_array_loop (N : usize) (n : nat) (a : array u32 N) (i : usize) (s : u32) : result u32 := match n with @@ -88,13 +88,13 @@ Fixpoint sum_array_loop . (** [loops::sum_array]: - Source: 'tests/src/loops.rs', lines 50:0-50:52 *) + Source: 'tests/src/loops.rs', lines 53:0-53:52 *) Definition sum_array (N : usize) (n : nat) (a : array u32 N) : result u32 := sum_array_loop N n a 0%usize 0%u32 . (** [loops::clear]: loop 0: - Source: 'tests/src/loops.rs', lines 62:0-68:1 *) + Source: 'tests/src/loops.rs', lines 65:0-71:1 *) Fixpoint clear_loop (n : nat) (v : alloc_vec_Vec u32) (i : usize) : result (alloc_vec_Vec u32) := match n with @@ -115,14 +115,14 @@ Fixpoint clear_loop . (** [loops::clear]: - Source: 'tests/src/loops.rs', lines 62:0-62:30 *) + Source: 'tests/src/loops.rs', lines 65:0-65:30 *) Definition clear (n : nat) (v : alloc_vec_Vec u32) : result (alloc_vec_Vec u32) := clear_loop n v 0%usize . (** [loops::List] - Source: 'tests/src/loops.rs', lines 70:0-70:16 *) + Source: 'tests/src/loops.rs', lines 73:0-73:16 *) Inductive List_t (T : Type) := | List_Cons : T -> List_t T -> List_t T | List_Nil : List_t T @@ -132,7 +132,7 @@ Arguments List_Cons { _ }. Arguments List_Nil { _ }. (** [loops::list_mem]: loop 0: - Source: 'tests/src/loops.rs', lines 76:0-85:1 *) + Source: 'tests/src/loops.rs', lines 79:0-88:1 *) Fixpoint list_mem_loop (n : nat) (x : u32) (ls : List_t u32) : result bool := match n with | O => Fail_ OutOfFuel @@ -145,13 +145,13 @@ Fixpoint list_mem_loop (n : nat) (x : u32) (ls : List_t u32) : result bool := . (** [loops::list_mem]: - Source: 'tests/src/loops.rs', lines 76:0-76:52 *) + Source: 'tests/src/loops.rs', lines 79:0-79:52 *) Definition list_mem (n : nat) (x : u32) (ls : List_t u32) : result bool := list_mem_loop n x ls . (** [loops::list_nth_mut_loop]: loop 0: - Source: 'tests/src/loops.rs', lines 88:0-98:1 *) + Source: 'tests/src/loops.rs', lines 91:0-101:1 *) Fixpoint list_nth_mut_loop_loop (T : Type) (n : nat) (ls : List_t T) (i : u32) : result (T * (T -> result (List_t T))) @@ -175,7 +175,7 @@ Fixpoint list_nth_mut_loop_loop . (** [loops::list_nth_mut_loop]: - Source: 'tests/src/loops.rs', lines 88:0-88:71 *) + Source: 'tests/src/loops.rs', lines 91:0-91:71 *) Definition list_nth_mut_loop (T : Type) (n : nat) (ls : List_t T) (i : u32) : result (T * (T -> result (List_t T))) @@ -184,7 +184,7 @@ Definition list_nth_mut_loop . (** [loops::list_nth_shared_loop]: loop 0: - Source: 'tests/src/loops.rs', lines 101:0-111:1 *) + Source: 'tests/src/loops.rs', lines 104:0-114:1 *) Fixpoint list_nth_shared_loop_loop (T : Type) (n : nat) (ls : List_t T) (i : u32) : result T := match n with @@ -201,14 +201,14 @@ Fixpoint list_nth_shared_loop_loop . (** [loops::list_nth_shared_loop]: - Source: 'tests/src/loops.rs', lines 101:0-101:66 *) + Source: 'tests/src/loops.rs', lines 104:0-104:66 *) Definition list_nth_shared_loop (T : Type) (n : nat) (ls : List_t T) (i : u32) : result T := list_nth_shared_loop_loop T n ls i . (** [loops::get_elem_mut]: loop 0: - Source: 'tests/src/loops.rs', lines 113:0-127:1 *) + Source: 'tests/src/loops.rs', lines 116:0-130:1 *) Fixpoint get_elem_mut_loop (n : nat) (x : usize) (ls : List_t usize) : result (usize * (usize -> result (List_t usize))) @@ -233,7 +233,7 @@ Fixpoint get_elem_mut_loop . (** [loops::get_elem_mut]: - Source: 'tests/src/loops.rs', lines 113:0-113:73 *) + Source: 'tests/src/loops.rs', lines 116:0-116:73 *) Definition get_elem_mut (n : nat) (slots : alloc_vec_Vec (List_t usize)) (x : usize) : result (usize * (usize -> result (alloc_vec_Vec (List_t usize)))) @@ -249,7 +249,7 @@ Definition get_elem_mut . (** [loops::get_elem_shared]: loop 0: - Source: 'tests/src/loops.rs', lines 129:0-143:1 *) + Source: 'tests/src/loops.rs', lines 132:0-146:1 *) Fixpoint get_elem_shared_loop (n : nat) (x : usize) (ls : List_t usize) : result usize := match n with @@ -263,7 +263,7 @@ Fixpoint get_elem_shared_loop . (** [loops::get_elem_shared]: - Source: 'tests/src/loops.rs', lines 129:0-129:68 *) + Source: 'tests/src/loops.rs', lines 132:0-132:68 *) Definition get_elem_shared (n : nat) (slots : alloc_vec_Vec (List_t usize)) (x : usize) : result usize @@ -275,7 +275,7 @@ Definition get_elem_shared . (** [loops::id_mut]: - Source: 'tests/src/loops.rs', lines 145:0-145:50 *) + Source: 'tests/src/loops.rs', lines 148:0-148:50 *) Definition id_mut (T : Type) (ls : List_t T) : result ((List_t T) * (List_t T -> result (List_t T))) @@ -284,12 +284,12 @@ Definition id_mut . (** [loops::id_shared]: - Source: 'tests/src/loops.rs', lines 149:0-149:45 *) + Source: 'tests/src/loops.rs', lines 152:0-152:45 *) Definition id_shared (T : Type) (ls : List_t T) : result (List_t T) := Ok ls. (** [loops::list_nth_mut_loop_with_id]: loop 0: - Source: 'tests/src/loops.rs', lines 154:0-165:1 *) + Source: 'tests/src/loops.rs', lines 157:0-168:1 *) Fixpoint list_nth_mut_loop_with_id_loop (T : Type) (n : nat) (i : u32) (ls : List_t T) : result (T * (T -> result (List_t T))) @@ -313,7 +313,7 @@ Fixpoint list_nth_mut_loop_with_id_loop . (** [loops::list_nth_mut_loop_with_id]: - Source: 'tests/src/loops.rs', lines 154:0-154:75 *) + Source: 'tests/src/loops.rs', lines 157:0-157:75 *) Definition list_nth_mut_loop_with_id (T : Type) (n : nat) (ls : List_t T) (i : u32) : result (T * (T -> result (List_t T))) @@ -327,7 +327,7 @@ Definition list_nth_mut_loop_with_id . (** [loops::list_nth_shared_loop_with_id]: loop 0: - Source: 'tests/src/loops.rs', lines 168:0-179:1 *) + Source: 'tests/src/loops.rs', lines 171:0-182:1 *) Fixpoint list_nth_shared_loop_with_id_loop (T : Type) (n : nat) (i : u32) (ls : List_t T) : result T := match n with @@ -345,14 +345,14 @@ Fixpoint list_nth_shared_loop_with_id_loop . (** [loops::list_nth_shared_loop_with_id]: - Source: 'tests/src/loops.rs', lines 168:0-168:70 *) + Source: 'tests/src/loops.rs', lines 171:0-171:70 *) Definition list_nth_shared_loop_with_id (T : Type) (n : nat) (ls : List_t T) (i : u32) : result T := ls1 <- id_shared T ls; list_nth_shared_loop_with_id_loop T n i ls1 . (** [loops::list_nth_mut_loop_pair]: loop 0: - Source: 'tests/src/loops.rs', lines 184:0-205:1 *) + Source: 'tests/src/loops.rs', lines 187:0-208:1 *) Fixpoint list_nth_mut_loop_pair_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T)) * (T -> result (List_t T))) @@ -386,7 +386,7 @@ Fixpoint list_nth_mut_loop_pair_loop . (** [loops::list_nth_mut_loop_pair]: - Source: 'tests/src/loops.rs', lines 184:0-188:27 *) + Source: 'tests/src/loops.rs', lines 187:0-191:27 *) Definition list_nth_mut_loop_pair (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T)) * (T -> result (List_t T))) @@ -395,7 +395,7 @@ Definition list_nth_mut_loop_pair . (** [loops::list_nth_shared_loop_pair]: loop 0: - Source: 'tests/src/loops.rs', lines 208:0-229:1 *) + Source: 'tests/src/loops.rs', lines 211:0-232:1 *) Fixpoint list_nth_shared_loop_pair_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result (T * T) @@ -419,7 +419,7 @@ Fixpoint list_nth_shared_loop_pair_loop . (** [loops::list_nth_shared_loop_pair]: - Source: 'tests/src/loops.rs', lines 208:0-212:19 *) + Source: 'tests/src/loops.rs', lines 211:0-215:19 *) Definition list_nth_shared_loop_pair (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result (T * T) @@ -428,7 +428,7 @@ Definition list_nth_shared_loop_pair . (** [loops::list_nth_mut_loop_pair_merge]: loop 0: - Source: 'tests/src/loops.rs', lines 233:0-248:1 *) + Source: 'tests/src/loops.rs', lines 236:0-251:1 *) Fixpoint list_nth_mut_loop_pair_merge_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * ((T * T) -> result ((List_t T) * (List_t T)))) @@ -464,7 +464,7 @@ Fixpoint list_nth_mut_loop_pair_merge_loop . (** [loops::list_nth_mut_loop_pair_merge]: - Source: 'tests/src/loops.rs', lines 233:0-237:27 *) + Source: 'tests/src/loops.rs', lines 236:0-240:27 *) Definition list_nth_mut_loop_pair_merge (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * ((T * T) -> result ((List_t T) * (List_t T)))) @@ -473,7 +473,7 @@ Definition list_nth_mut_loop_pair_merge . (** [loops::list_nth_shared_loop_pair_merge]: loop 0: - Source: 'tests/src/loops.rs', lines 251:0-266:1 *) + Source: 'tests/src/loops.rs', lines 254:0-269:1 *) Fixpoint list_nth_shared_loop_pair_merge_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result (T * T) @@ -498,7 +498,7 @@ Fixpoint list_nth_shared_loop_pair_merge_loop . (** [loops::list_nth_shared_loop_pair_merge]: - Source: 'tests/src/loops.rs', lines 251:0-255:19 *) + Source: 'tests/src/loops.rs', lines 254:0-258:19 *) Definition list_nth_shared_loop_pair_merge (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result (T * T) @@ -507,7 +507,7 @@ Definition list_nth_shared_loop_pair_merge . (** [loops::list_nth_mut_shared_loop_pair]: loop 0: - Source: 'tests/src/loops.rs', lines 269:0-284:1 *) + Source: 'tests/src/loops.rs', lines 272:0-287:1 *) Fixpoint list_nth_mut_shared_loop_pair_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -538,7 +538,7 @@ Fixpoint list_nth_mut_shared_loop_pair_loop . (** [loops::list_nth_mut_shared_loop_pair]: - Source: 'tests/src/loops.rs', lines 269:0-273:23 *) + Source: 'tests/src/loops.rs', lines 272:0-276:23 *) Definition list_nth_mut_shared_loop_pair (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -547,7 +547,7 @@ Definition list_nth_mut_shared_loop_pair . (** [loops::list_nth_mut_shared_loop_pair_merge]: loop 0: - Source: 'tests/src/loops.rs', lines 288:0-303:1 *) + Source: 'tests/src/loops.rs', lines 291:0-306:1 *) Fixpoint list_nth_mut_shared_loop_pair_merge_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -578,7 +578,7 @@ Fixpoint list_nth_mut_shared_loop_pair_merge_loop . (** [loops::list_nth_mut_shared_loop_pair_merge]: - Source: 'tests/src/loops.rs', lines 288:0-292:23 *) + Source: 'tests/src/loops.rs', lines 291:0-295:23 *) Definition list_nth_mut_shared_loop_pair_merge (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -587,7 +587,7 @@ Definition list_nth_mut_shared_loop_pair_merge . (** [loops::list_nth_shared_mut_loop_pair]: loop 0: - Source: 'tests/src/loops.rs', lines 307:0-322:1 *) + Source: 'tests/src/loops.rs', lines 310:0-325:1 *) Fixpoint list_nth_shared_mut_loop_pair_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -618,7 +618,7 @@ Fixpoint list_nth_shared_mut_loop_pair_loop . (** [loops::list_nth_shared_mut_loop_pair]: - Source: 'tests/src/loops.rs', lines 307:0-311:23 *) + Source: 'tests/src/loops.rs', lines 310:0-314:23 *) Definition list_nth_shared_mut_loop_pair (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -627,7 +627,7 @@ Definition list_nth_shared_mut_loop_pair . (** [loops::list_nth_shared_mut_loop_pair_merge]: loop 0: - Source: 'tests/src/loops.rs', lines 326:0-341:1 *) + Source: 'tests/src/loops.rs', lines 329:0-344:1 *) Fixpoint list_nth_shared_mut_loop_pair_merge_loop (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -658,7 +658,7 @@ Fixpoint list_nth_shared_mut_loop_pair_merge_loop . (** [loops::list_nth_shared_mut_loop_pair_merge]: - Source: 'tests/src/loops.rs', lines 326:0-330:23 *) + Source: 'tests/src/loops.rs', lines 329:0-333:23 *) Definition list_nth_shared_mut_loop_pair_merge (T : Type) (n : nat) (ls0 : List_t T) (ls1 : List_t T) (i : u32) : result ((T * T) * (T -> result (List_t T))) @@ -667,7 +667,7 @@ Definition list_nth_shared_mut_loop_pair_merge . (** [loops::ignore_input_mut_borrow]: loop 0: - Source: 'tests/src/loops.rs', lines 345:0-349:1 *) + Source: 'tests/src/loops.rs', lines 348:0-352:1 *) Fixpoint ignore_input_mut_borrow_loop (n : nat) (i : u32) : result unit := match n with | O => Fail_ OutOfFuel @@ -679,14 +679,14 @@ Fixpoint ignore_input_mut_borrow_loop (n : nat) (i : u32) : result unit := . (** [loops::ignore_input_mut_borrow]: - Source: 'tests/src/loops.rs', lines 345:0-345:56 *) + Source: 'tests/src/loops.rs', lines 348:0-348:56 *) Definition ignore_input_mut_borrow (n : nat) (_a : u32) (i : u32) : result u32 := _ <- ignore_input_mut_borrow_loop n i; Ok _a . (** [loops::incr_ignore_input_mut_borrow]: loop 0: - Source: 'tests/src/loops.rs', lines 353:0-358:1 *) + Source: 'tests/src/loops.rs', lines 356:0-361:1 *) Fixpoint incr_ignore_input_mut_borrow_loop (n : nat) (i : u32) : result unit := match n with | O => Fail_ OutOfFuel @@ -698,14 +698,14 @@ Fixpoint incr_ignore_input_mut_borrow_loop (n : nat) (i : u32) : result unit := . (** [loops::incr_ignore_input_mut_borrow]: - Source: 'tests/src/loops.rs', lines 353:0-353:60 *) + Source: 'tests/src/loops.rs', lines 356:0-356:60 *) Definition incr_ignore_input_mut_borrow (n : nat) (a : u32) (i : u32) : result u32 := a1 <- u32_add a 1%u32; _ <- incr_ignore_input_mut_borrow_loop n i; Ok a1 . (** [loops::ignore_input_shared_borrow]: loop 0: - Source: 'tests/src/loops.rs', lines 362:0-366:1 *) + Source: 'tests/src/loops.rs', lines 365:0-369:1 *) Fixpoint ignore_input_shared_borrow_loop (n : nat) (i : u32) : result unit := match n with | O => Fail_ OutOfFuel @@ -717,7 +717,7 @@ Fixpoint ignore_input_shared_borrow_loop (n : nat) (i : u32) : result unit := . (** [loops::ignore_input_shared_borrow]: - Source: 'tests/src/loops.rs', lines 362:0-362:59 *) + Source: 'tests/src/loops.rs', lines 365:0-365:59 *) Definition ignore_input_shared_borrow (n : nat) (_a : u32) (i : u32) : result u32 := _ <- ignore_input_shared_borrow_loop n i; Ok _a diff --git a/tests/coq/misc/NoNestedBorrows.v b/tests/coq/misc/NoNestedBorrows.v index a83347a7..434b820c 100644 --- a/tests/coq/misc/NoNestedBorrows.v +++ b/tests/coq/misc/NoNestedBorrows.v @@ -9,7 +9,7 @@ Local Open Scope Primitives_scope. Module NoNestedBorrows. (** [no_nested_borrows::Pair] - Source: 'tests/src/no_nested_borrows.rs', lines 4:0-4:23 *) + Source: 'tests/src/no_nested_borrows.rs', lines 6:0-6:23 *) Record Pair_t (T1 T2 : Type) := mkPair_t { pair_x : T1; pair_y : T2; }. Arguments mkPair_t { _ _ }. @@ -17,7 +17,7 @@ Arguments pair_x { _ _ }. Arguments pair_y { _ _ }. (** [no_nested_borrows::List] - Source: 'tests/src/no_nested_borrows.rs', lines 9:0-9:16 *) + Source: 'tests/src/no_nested_borrows.rs', lines 11:0-11:16 *) Inductive List_t (T : Type) := | List_Cons : T -> List_t T -> List_t T | List_Nil : List_t T @@ -27,25 +27,25 @@ Arguments List_Cons { _ }. Arguments List_Nil { _ }. (** [no_nested_borrows::One] - Source: 'tests/src/no_nested_borrows.rs', lines 20:0-20:16 *) + Source: 'tests/src/no_nested_borrows.rs', lines 22:0-22:16 *) Inductive One_t (T1 : Type) := | One_One : T1 -> One_t T1. Arguments One_One { _ }. (** [no_nested_borrows::EmptyEnum] - Source: 'tests/src/no_nested_borrows.rs', lines 26:0-26:18 *) + Source: 'tests/src/no_nested_borrows.rs', lines 28:0-28:18 *) Inductive EmptyEnum_t := | EmptyEnum_Empty : EmptyEnum_t. (** [no_nested_borrows::Enum] - Source: 'tests/src/no_nested_borrows.rs', lines 32:0-32:13 *) + Source: 'tests/src/no_nested_borrows.rs', lines 34:0-34:13 *) Inductive Enum_t := | Enum_Variant1 : Enum_t | Enum_Variant2 : Enum_t. (** [no_nested_borrows::EmptyStruct] - Source: 'tests/src/no_nested_borrows.rs', lines 39:0-39:22 *) + Source: 'tests/src/no_nested_borrows.rs', lines 41:0-41:22 *) Definition EmptyStruct_t : Type := unit. (** [no_nested_borrows::Sum] - Source: 'tests/src/no_nested_borrows.rs', lines 41:0-41:20 *) + Source: 'tests/src/no_nested_borrows.rs', lines 43:0-43:20 *) Inductive Sum_t (T1 T2 : Type) := | Sum_Left : T1 -> Sum_t T1 T2 | Sum_Right : T2 -> Sum_t T1 T2 @@ -55,22 +55,22 @@ Arguments Sum_Left { _ _ }. Arguments Sum_Right { _ _ }. (** [no_nested_borrows::cast_u32_to_i32]: - Source: 'tests/src/no_nested_borrows.rs', lines 46:0-46:37 *) + Source: 'tests/src/no_nested_borrows.rs', lines 48:0-48:37 *) Definition cast_u32_to_i32 (x : u32) : result i32 := scalar_cast U32 I32 x. (** [no_nested_borrows::cast_bool_to_i32]: - Source: 'tests/src/no_nested_borrows.rs', lines 50:0-50:39 *) + Source: 'tests/src/no_nested_borrows.rs', lines 52:0-52:39 *) Definition cast_bool_to_i32 (x : bool) : result i32 := scalar_cast_bool I32 x. (** [no_nested_borrows::cast_bool_to_bool]: - Source: 'tests/src/no_nested_borrows.rs', lines 55:0-55:41 *) + Source: 'tests/src/no_nested_borrows.rs', lines 57:0-57:41 *) Definition cast_bool_to_bool (x : bool) : result bool := Ok x. (** [no_nested_borrows::test2]: - Source: 'tests/src/no_nested_borrows.rs', lines 60:0-60:14 *) + Source: 'tests/src/no_nested_borrows.rs', lines 62:0-62:14 *) Definition test2 : result unit := _ <- u32_add 23%u32 44%u32; Ok tt. @@ -78,13 +78,13 @@ Definition test2 : result unit := Check (test2 )%return. (** [no_nested_borrows::get_max]: - Source: 'tests/src/no_nested_borrows.rs', lines 72:0-72:37 *) + Source: 'tests/src/no_nested_borrows.rs', lines 74:0-74:37 *) Definition get_max (x : u32) (y : u32) : result u32 := if x s>= y then Ok x else Ok y . (** [no_nested_borrows::test3]: - Source: 'tests/src/no_nested_borrows.rs', lines 80:0-80:14 *) + Source: 'tests/src/no_nested_borrows.rs', lines 82:0-82:14 *) Definition test3 : result unit := x <- get_max 4%u32 3%u32; y <- get_max 10%u32 11%u32; @@ -96,7 +96,7 @@ Definition test3 : result unit := Check (test3 )%return. (** [no_nested_borrows::test_neg1]: - Source: 'tests/src/no_nested_borrows.rs', lines 87:0-87:18 *) + Source: 'tests/src/no_nested_borrows.rs', lines 89:0-89:18 *) Definition test_neg1 : result unit := y <- i32_neg 3%i32; if negb (y s= (-3)%i32) then Fail_ Failure else Ok tt . @@ -105,7 +105,7 @@ Definition test_neg1 : result unit := Check (test_neg1 )%return. (** [no_nested_borrows::refs_test1]: - Source: 'tests/src/no_nested_borrows.rs', lines 94:0-94:19 *) + Source: 'tests/src/no_nested_borrows.rs', lines 96:0-96:19 *) Definition refs_test1 : result unit := if negb (1%i32 s= 1%i32) then Fail_ Failure else Ok tt . @@ -114,7 +114,7 @@ Definition refs_test1 : result unit := Check (refs_test1 )%return. (** [no_nested_borrows::refs_test2]: - Source: 'tests/src/no_nested_borrows.rs', lines 105:0-105:19 *) + Source: 'tests/src/no_nested_borrows.rs', lines 107:0-107:19 *) Definition refs_test2 : result unit := if negb (2%i32 s= 2%i32) then Fail_ Failure @@ -131,7 +131,7 @@ Definition refs_test2 : result unit := Check (refs_test2 )%return. (** [no_nested_borrows::test_list1]: - Source: 'tests/src/no_nested_borrows.rs', lines 121:0-121:19 *) + Source: 'tests/src/no_nested_borrows.rs', lines 123:0-123:19 *) Definition test_list1 : result unit := Ok tt. @@ -139,7 +139,7 @@ Definition test_list1 : result unit := Check (test_list1 )%return. (** [no_nested_borrows::test_box1]: - Source: 'tests/src/no_nested_borrows.rs', lines 126:0-126:18 *) + Source: 'tests/src/no_nested_borrows.rs', lines 128:0-128:18 *) Definition test_box1 : result unit := p <- alloc_boxed_Box_deref_mut i32 0%i32; let (_, deref_mut_back) := p in @@ -152,24 +152,24 @@ Definition test_box1 : result unit := Check (test_box1 )%return. (** [no_nested_borrows::copy_int]: - Source: 'tests/src/no_nested_borrows.rs', lines 136:0-136:30 *) + Source: 'tests/src/no_nested_borrows.rs', lines 138:0-138:30 *) Definition copy_int (x : i32) : result i32 := Ok x. (** [no_nested_borrows::test_unreachable]: - Source: 'tests/src/no_nested_borrows.rs', lines 142:0-142:32 *) + Source: 'tests/src/no_nested_borrows.rs', lines 144:0-144:32 *) Definition test_unreachable (b : bool) : result unit := if b then Fail_ Failure else Ok tt . (** [no_nested_borrows::test_panic]: - Source: 'tests/src/no_nested_borrows.rs', lines 150:0-150:26 *) + Source: 'tests/src/no_nested_borrows.rs', lines 152:0-152:26 *) Definition test_panic (b : bool) : result unit := if b then Fail_ Failure else Ok tt . (** [no_nested_borrows::test_copy_int]: - Source: 'tests/src/no_nested_borrows.rs', lines 157:0-157:22 *) + Source: 'tests/src/no_nested_borrows.rs', lines 159:0-159:22 *) Definition test_copy_int : result unit := y <- copy_int 0%i32; if negb (0%i32 s= y) then Fail_ Failure else Ok tt . @@ -178,13 +178,13 @@ Definition test_copy_int : result unit := Check (test_copy_int )%return. (** [no_nested_borrows::is_cons]: - Source: 'tests/src/no_nested_borrows.rs', lines 164:0-164:38 *) + Source: 'tests/src/no_nested_borrows.rs', lines 166:0-166:38 *) Definition is_cons (T : Type) (l : List_t T) : result bool := match l with | List_Cons _ _ => Ok true | List_Nil => Ok false end . (** [no_nested_borrows::test_is_cons]: - Source: 'tests/src/no_nested_borrows.rs', lines 171:0-171:21 *) + Source: 'tests/src/no_nested_borrows.rs', lines 173:0-173:21 *) Definition test_is_cons : result unit := b <- is_cons i32 (List_Cons 0%i32 List_Nil); if negb b then Fail_ Failure else Ok tt @@ -194,13 +194,13 @@ Definition test_is_cons : result unit := Check (test_is_cons )%return. (** [no_nested_borrows::split_list]: - Source: 'tests/src/no_nested_borrows.rs', lines 177:0-177:48 *) + Source: 'tests/src/no_nested_borrows.rs', lines 179:0-179:48 *) Definition split_list (T : Type) (l : List_t T) : result (T * (List_t T)) := match l with | List_Cons hd tl => Ok (hd, tl) | List_Nil => Fail_ Failure end . (** [no_nested_borrows::test_split_list]: - Source: 'tests/src/no_nested_borrows.rs', lines 185:0-185:24 *) + Source: 'tests/src/no_nested_borrows.rs', lines 187:0-187:24 *) Definition test_split_list : result unit := p <- split_list i32 (List_Cons 0%i32 List_Nil); let (hd, _) := p in @@ -211,7 +211,7 @@ Definition test_split_list : result unit := Check (test_split_list )%return. (** [no_nested_borrows::choose]: - Source: 'tests/src/no_nested_borrows.rs', lines 192:0-192:70 *) + Source: 'tests/src/no_nested_borrows.rs', lines 194:0-194:70 *) Definition choose (T : Type) (b : bool) (x : T) (y : T) : result (T * (T -> result (T * T))) := if b @@ -220,7 +220,7 @@ Definition choose . (** [no_nested_borrows::choose_test]: - Source: 'tests/src/no_nested_borrows.rs', lines 200:0-200:20 *) + Source: 'tests/src/no_nested_borrows.rs', lines 202:0-202:20 *) Definition choose_test : result unit := p <- choose i32 true 0%i32 0%i32; let (z, choose_back) := p in @@ -239,18 +239,18 @@ Definition choose_test : result unit := Check (choose_test )%return. (** [no_nested_borrows::test_char]: - Source: 'tests/src/no_nested_borrows.rs', lines 212:0-212:26 *) + Source: 'tests/src/no_nested_borrows.rs', lines 214:0-214:26 *) Definition test_char : result char := Ok (char_of_byte Coq.Init.Byte.x61). (** [no_nested_borrows::Tree] - Source: 'tests/src/no_nested_borrows.rs', lines 217:0-217:16 *) + Source: 'tests/src/no_nested_borrows.rs', lines 219:0-219:16 *) Inductive Tree_t (T : Type) := | Tree_Leaf : T -> Tree_t T | Tree_Node : T -> NodeElem_t T -> Tree_t T -> Tree_t T (** [no_nested_borrows::NodeElem] - Source: 'tests/src/no_nested_borrows.rs', lines 222:0-222:20 *) + Source: 'tests/src/no_nested_borrows.rs', lines 224:0-224:20 *) with NodeElem_t (T : Type) := | NodeElem_Cons : Tree_t T -> NodeElem_t T -> NodeElem_t T | NodeElem_Nil : NodeElem_t T @@ -263,7 +263,7 @@ Arguments NodeElem_Cons { _ }. Arguments NodeElem_Nil { _ }. (** [no_nested_borrows::list_length]: - Source: 'tests/src/no_nested_borrows.rs', lines 257:0-257:48 *) + Source: 'tests/src/no_nested_borrows.rs', lines 259:0-259:48 *) Fixpoint list_length (T : Type) (l : List_t T) : result u32 := match l with | List_Cons _ l1 => i <- list_length T l1; u32_add 1%u32 i @@ -272,7 +272,7 @@ Fixpoint list_length (T : Type) (l : List_t T) : result u32 := . (** [no_nested_borrows::list_nth_shared]: - Source: 'tests/src/no_nested_borrows.rs', lines 265:0-265:62 *) + Source: 'tests/src/no_nested_borrows.rs', lines 267:0-267:62 *) Fixpoint list_nth_shared (T : Type) (l : List_t T) (i : u32) : result T := match l with | List_Cons x tl => @@ -284,7 +284,7 @@ Fixpoint list_nth_shared (T : Type) (l : List_t T) (i : u32) : result T := . (** [no_nested_borrows::list_nth_mut]: - Source: 'tests/src/no_nested_borrows.rs', lines 281:0-281:67 *) + Source: 'tests/src/no_nested_borrows.rs', lines 283:0-283:67 *) Fixpoint list_nth_mut (T : Type) (l : List_t T) (i : u32) : result (T * (T -> result (List_t T))) @@ -305,7 +305,7 @@ Fixpoint list_nth_mut . (** [no_nested_borrows::list_rev_aux]: - Source: 'tests/src/no_nested_borrows.rs', lines 297:0-297:63 *) + Source: 'tests/src/no_nested_borrows.rs', lines 299:0-299:63 *) Fixpoint list_rev_aux (T : Type) (li : List_t T) (lo : List_t T) : result (List_t T) := match li with @@ -315,14 +315,14 @@ Fixpoint list_rev_aux . (** [no_nested_borrows::list_rev]: - Source: 'tests/src/no_nested_borrows.rs', lines 311:0-311:42 *) + Source: 'tests/src/no_nested_borrows.rs', lines 313:0-313:42 *) Definition list_rev (T : Type) (l : List_t T) : result (List_t T) := let (li, _) := core_mem_replace (List_t T) l List_Nil in list_rev_aux T li List_Nil . (** [no_nested_borrows::test_list_functions]: - Source: 'tests/src/no_nested_borrows.rs', lines 316:0-316:28 *) + Source: 'tests/src/no_nested_borrows.rs', lines 318:0-318:28 *) Definition test_list_functions : result unit := let l := List_Cons 2%i32 List_Nil in let l1 := List_Cons 1%i32 l in @@ -361,7 +361,7 @@ Definition test_list_functions : result unit := Check (test_list_functions )%return. (** [no_nested_borrows::id_mut_pair1]: - Source: 'tests/src/no_nested_borrows.rs', lines 332:0-332:89 *) + Source: 'tests/src/no_nested_borrows.rs', lines 334:0-334:89 *) Definition id_mut_pair1 (T1 T2 : Type) (x : T1) (y : T2) : result ((T1 * T2) * ((T1 * T2) -> result (T1 * T2))) @@ -370,7 +370,7 @@ Definition id_mut_pair1 . (** [no_nested_borrows::id_mut_pair2]: - Source: 'tests/src/no_nested_borrows.rs', lines 336:0-336:88 *) + Source: 'tests/src/no_nested_borrows.rs', lines 338:0-338:88 *) Definition id_mut_pair2 (T1 T2 : Type) (p : (T1 * T2)) : result ((T1 * T2) * ((T1 * T2) -> result (T1 * T2))) @@ -379,7 +379,7 @@ Definition id_mut_pair2 . (** [no_nested_borrows::id_mut_pair3]: - Source: 'tests/src/no_nested_borrows.rs', lines 340:0-340:93 *) + Source: 'tests/src/no_nested_borrows.rs', lines 342:0-342:93 *) Definition id_mut_pair3 (T1 T2 : Type) (x : T1) (y : T2) : result ((T1 * T2) * (T1 -> result T1) * (T2 -> result T2)) @@ -388,7 +388,7 @@ Definition id_mut_pair3 . (** [no_nested_borrows::id_mut_pair4]: - Source: 'tests/src/no_nested_borrows.rs', lines 344:0-344:92 *) + Source: 'tests/src/no_nested_borrows.rs', lines 346:0-346:92 *) Definition id_mut_pair4 (T1 T2 : Type) (p : (T1 * T2)) : result ((T1 * T2) * (T1 -> result T1) * (T2 -> result T2)) @@ -397,7 +397,7 @@ Definition id_mut_pair4 . (** [no_nested_borrows::StructWithTuple] - Source: 'tests/src/no_nested_borrows.rs', lines 351:0-351:34 *) + Source: 'tests/src/no_nested_borrows.rs', lines 353:0-353:34 *) Record StructWithTuple_t (T1 T2 : Type) := mkStructWithTuple_t { structWithTuple_p : (T1 * T2); @@ -408,25 +408,25 @@ Arguments mkStructWithTuple_t { _ _ }. Arguments structWithTuple_p { _ _ }. (** [no_nested_borrows::new_tuple1]: - Source: 'tests/src/no_nested_borrows.rs', lines 355:0-355:48 *) + Source: 'tests/src/no_nested_borrows.rs', lines 357:0-357:48 *) Definition new_tuple1 : result (StructWithTuple_t u32 u32) := Ok {| structWithTuple_p := (1%u32, 2%u32) |} . (** [no_nested_borrows::new_tuple2]: - Source: 'tests/src/no_nested_borrows.rs', lines 359:0-359:48 *) + Source: 'tests/src/no_nested_borrows.rs', lines 361:0-361:48 *) Definition new_tuple2 : result (StructWithTuple_t i16 i16) := Ok {| structWithTuple_p := (1%i16, 2%i16) |} . (** [no_nested_borrows::new_tuple3]: - Source: 'tests/src/no_nested_borrows.rs', lines 363:0-363:48 *) + Source: 'tests/src/no_nested_borrows.rs', lines 365:0-365:48 *) Definition new_tuple3 : result (StructWithTuple_t u64 i64) := Ok {| structWithTuple_p := (1%u64, 2%i64) |} . (** [no_nested_borrows::StructWithPair] - Source: 'tests/src/no_nested_borrows.rs', lines 368:0-368:33 *) + Source: 'tests/src/no_nested_borrows.rs', lines 370:0-370:33 *) Record StructWithPair_t (T1 T2 : Type) := mkStructWithPair_t { structWithPair_p : Pair_t T1 T2; @@ -437,13 +437,13 @@ Arguments mkStructWithPair_t { _ _ }. Arguments structWithPair_p { _ _ }. (** [no_nested_borrows::new_pair1]: - Source: 'tests/src/no_nested_borrows.rs', lines 372:0-372:46 *) + Source: 'tests/src/no_nested_borrows.rs', lines 374:0-374:46 *) Definition new_pair1 : result (StructWithPair_t u32 u32) := Ok {| structWithPair_p := {| pair_x := 1%u32; pair_y := 2%u32 |} |} . (** [no_nested_borrows::test_constants]: - Source: 'tests/src/no_nested_borrows.rs', lines 380:0-380:23 *) + Source: 'tests/src/no_nested_borrows.rs', lines 382:0-382:23 *) Definition test_constants : result unit := swt <- new_tuple1; let (i, _) := swt.(structWithTuple_p) in @@ -470,7 +470,7 @@ Definition test_constants : result unit := Check (test_constants )%return. (** [no_nested_borrows::test_weird_borrows1]: - Source: 'tests/src/no_nested_borrows.rs', lines 389:0-389:28 *) + Source: 'tests/src/no_nested_borrows.rs', lines 391:0-391:28 *) Definition test_weird_borrows1 : result unit := Ok tt. @@ -478,78 +478,78 @@ Definition test_weird_borrows1 : result unit := Check (test_weird_borrows1 )%return. (** [no_nested_borrows::test_mem_replace]: - Source: 'tests/src/no_nested_borrows.rs', lines 399:0-399:37 *) + Source: 'tests/src/no_nested_borrows.rs', lines 401:0-401:37 *) Definition test_mem_replace (px : u32) : result u32 := let (y, _) := core_mem_replace u32 px 1%u32 in if negb (y s= 0%u32) then Fail_ Failure else Ok 2%u32 . (** [no_nested_borrows::test_shared_borrow_bool1]: - Source: 'tests/src/no_nested_borrows.rs', lines 406:0-406:47 *) + Source: 'tests/src/no_nested_borrows.rs', lines 408:0-408:47 *) Definition test_shared_borrow_bool1 (b : bool) : result u32 := if b then Ok 0%u32 else Ok 1%u32 . (** [no_nested_borrows::test_shared_borrow_bool2]: - Source: 'tests/src/no_nested_borrows.rs', lines 419:0-419:40 *) + Source: 'tests/src/no_nested_borrows.rs', lines 421:0-421:40 *) Definition test_shared_borrow_bool2 : result u32 := Ok 0%u32. (** [no_nested_borrows::test_shared_borrow_enum1]: - Source: 'tests/src/no_nested_borrows.rs', lines 434:0-434:52 *) + Source: 'tests/src/no_nested_borrows.rs', lines 436:0-436:52 *) Definition test_shared_borrow_enum1 (l : List_t u32) : result u32 := match l with | List_Cons _ _ => Ok 1%u32 | List_Nil => Ok 0%u32 end . (** [no_nested_borrows::test_shared_borrow_enum2]: - Source: 'tests/src/no_nested_borrows.rs', lines 446:0-446:40 *) + Source: 'tests/src/no_nested_borrows.rs', lines 448:0-448:40 *) Definition test_shared_borrow_enum2 : result u32 := Ok 0%u32. (** [no_nested_borrows::incr]: - Source: 'tests/src/no_nested_borrows.rs', lines 457:0-457:24 *) + Source: 'tests/src/no_nested_borrows.rs', lines 459:0-459:24 *) Definition incr (x : u32) : result u32 := u32_add x 1%u32. (** [no_nested_borrows::call_incr]: - Source: 'tests/src/no_nested_borrows.rs', lines 461:0-461:35 *) + Source: 'tests/src/no_nested_borrows.rs', lines 463:0-463:35 *) Definition call_incr (x : u32) : result u32 := incr x. (** [no_nested_borrows::read_then_incr]: - Source: 'tests/src/no_nested_borrows.rs', lines 466:0-466:41 *) + Source: 'tests/src/no_nested_borrows.rs', lines 468:0-468:41 *) Definition read_then_incr (x : u32) : result (u32 * u32) := x1 <- u32_add x 1%u32; Ok (x, x1) . (** [no_nested_borrows::Tuple] - Source: 'tests/src/no_nested_borrows.rs', lines 472:0-472:24 *) + Source: 'tests/src/no_nested_borrows.rs', lines 474:0-474:24 *) Definition Tuple_t (T1 T2 : Type) : Type := T1 * T2. (** [no_nested_borrows::use_tuple_struct]: - Source: 'tests/src/no_nested_borrows.rs', lines 474:0-474:48 *) + Source: 'tests/src/no_nested_borrows.rs', lines 476:0-476:48 *) Definition use_tuple_struct (x : Tuple_t u32 u32) : result (Tuple_t u32 u32) := let (_, i) := x in Ok (1%u32, i) . (** [no_nested_borrows::create_tuple_struct]: - Source: 'tests/src/no_nested_borrows.rs', lines 478:0-478:61 *) + Source: 'tests/src/no_nested_borrows.rs', lines 480:0-480:61 *) Definition create_tuple_struct (x : u32) (y : u64) : result (Tuple_t u32 u64) := Ok (x, y) . (** [no_nested_borrows::IdType] - Source: 'tests/src/no_nested_borrows.rs', lines 483:0-483:20 *) + Source: 'tests/src/no_nested_borrows.rs', lines 485:0-485:20 *) Definition IdType_t (T : Type) : Type := T. (** [no_nested_borrows::use_id_type]: - Source: 'tests/src/no_nested_borrows.rs', lines 485:0-485:40 *) + Source: 'tests/src/no_nested_borrows.rs', lines 487:0-487:40 *) Definition use_id_type (T : Type) (x : IdType_t T) : result T := Ok x. (** [no_nested_borrows::create_id_type]: - Source: 'tests/src/no_nested_borrows.rs', lines 489:0-489:43 *) + Source: 'tests/src/no_nested_borrows.rs', lines 491:0-491:43 *) Definition create_id_type (T : Type) (x : T) : result (IdType_t T) := Ok x. diff --git a/tests/coq/misc/Paper.v b/tests/coq/misc/Paper.v index 661a8cc2..21e86542 100644 --- a/tests/coq/misc/Paper.v +++ b/tests/coq/misc/Paper.v @@ -9,12 +9,12 @@ Local Open Scope Primitives_scope. Module Paper. (** [paper::ref_incr]: - Source: 'tests/src/paper.rs', lines 4:0-4:28 *) + Source: 'tests/src/paper.rs', lines 6:0-6:28 *) Definition ref_incr (x : i32) : result i32 := i32_add x 1%i32. (** [paper::test_incr]: - Source: 'tests/src/paper.rs', lines 8:0-8:18 *) + Source: 'tests/src/paper.rs', lines 10:0-10:18 *) Definition test_incr : result unit := x <- ref_incr 0%i32; if negb (x s= 1%i32) then Fail_ Failure else Ok tt . @@ -23,7 +23,7 @@ Definition test_incr : result unit := Check (test_incr )%return. (** [paper::choose]: - Source: 'tests/src/paper.rs', lines 15:0-15:70 *) + Source: 'tests/src/paper.rs', lines 17:0-17:70 *) Definition choose (T : Type) (b : bool) (x : T) (y : T) : result (T * (T -> result (T * T))) := if b @@ -32,7 +32,7 @@ Definition choose . (** [paper::test_choose]: - Source: 'tests/src/paper.rs', lines 23:0-23:20 *) + Source: 'tests/src/paper.rs', lines 25:0-25:20 *) Definition test_choose : result unit := p <- choose i32 true 0%i32 0%i32; let (z, choose_back) := p in @@ -51,7 +51,7 @@ Definition test_choose : result unit := Check (test_choose )%return. (** [paper::List] - Source: 'tests/src/paper.rs', lines 35:0-35:16 *) + Source: 'tests/src/paper.rs', lines 37:0-37:16 *) Inductive List_t (T : Type) := | List_Cons : T -> List_t T -> List_t T | List_Nil : List_t T @@ -61,7 +61,7 @@ Arguments List_Cons { _ }. Arguments List_Nil { _ }. (** [paper::list_nth_mut]: - Source: 'tests/src/paper.rs', lines 42:0-42:67 *) + Source: 'tests/src/paper.rs', lines 44:0-44:67 *) Fixpoint list_nth_mut (T : Type) (l : List_t T) (i : u32) : result (T * (T -> result (List_t T))) @@ -82,7 +82,7 @@ Fixpoint list_nth_mut . (** [paper::sum]: - Source: 'tests/src/paper.rs', lines 57:0-57:32 *) + Source: 'tests/src/paper.rs', lines 59:0-59:32 *) Fixpoint sum (l : List_t i32) : result i32 := match l with | List_Cons x tl => i <- sum tl; i32_add x i @@ -91,7 +91,7 @@ Fixpoint sum (l : List_t i32) : result i32 := . (** [paper::test_nth]: - Source: 'tests/src/paper.rs', lines 68:0-68:17 *) + Source: 'tests/src/paper.rs', lines 70:0-70:17 *) Definition test_nth : result unit := let l := List_Cons 3%i32 List_Nil in let l1 := List_Cons 2%i32 l in @@ -107,7 +107,7 @@ Definition test_nth : result unit := Check (test_nth )%return. (** [paper::call_choose]: - Source: 'tests/src/paper.rs', lines 76:0-76:44 *) + Source: 'tests/src/paper.rs', lines 78:0-78:44 *) Definition call_choose (p : (u32 * u32)) : result u32 := let (px, py) := p in p1 <- choose u32 true px py; diff --git a/tests/coq/misc/PoloniusList.v b/tests/coq/misc/PoloniusList.v index c89f9655..91cfcdb7 100644 --- a/tests/coq/misc/PoloniusList.v +++ b/tests/coq/misc/PoloniusList.v @@ -9,7 +9,7 @@ Local Open Scope Primitives_scope. Module PoloniusList. (** [polonius_list::List] - Source: 'tests/src/polonius_list.rs', lines 3:0-3:16 *) + Source: 'tests/src/polonius_list.rs', lines 5:0-5:16 *) Inductive List_t (T : Type) := | List_Cons : T -> List_t T -> List_t T | List_Nil : List_t T @@ -19,7 +19,7 @@ Arguments List_Cons { _ }. Arguments List_Nil { _ }. (** [polonius_list::get_list_at_x]: - Source: 'tests/src/polonius_list.rs', lines 13:0-13:76 *) + Source: 'tests/src/polonius_list.rs', lines 15:0-15:76 *) Fixpoint get_list_at_x (ls : List_t u32) (x : u32) : result ((List_t u32) * (List_t u32 -> result (List_t u32))) -- cgit v1.2.3