summaryrefslogtreecommitdiff
path: root/tests/coq/misc/Paper.v
blob: e5728364b73535372d8362da7fc58a88784fe8b7 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
102
103
104
105
106
107
108
109
110
111
112
113
114
115
116
117
118
119
120
121
(** THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS *)
(** [paper] *)
Require Import Primitives.
Import Primitives.
Require Import Coq.ZArith.ZArith.
Require Import List.
Import ListNotations.
Local Open Scope Primitives_scope.
Module Paper.

(** [paper::ref_incr]:
    Source: 'tests/src/paper.rs', lines 7:0-7:28 *)
Definition ref_incr (x : i32) : result i32 :=
  i32_add x 1%i32.

(** [paper::test_incr]:
    Source: 'tests/src/paper.rs', lines 11:0-11:18 *)
Definition test_incr : result unit :=
  x <- ref_incr 0%i32; if negb (x s= 1%i32) then Fail_ Failure else Ok tt
.

(** Unit test for [paper::test_incr] *)
Check (test_incr )%return.

(** [paper::choose]:
    Source: 'tests/src/paper.rs', lines 18:0-18:70 *)
Definition choose
  (T : Type) (b : bool) (x : T) (y : T) : result (T * (T -> result (T * T))) :=
  if b
  then let back := fun (ret : T) => Ok (ret, y) in Ok (x, back)
  else let back := fun (ret : T) => Ok (x, ret) in Ok (y, back)
.

(** [paper::test_choose]:
    Source: 'tests/src/paper.rs', lines 26:0-26:20 *)
Definition test_choose : result unit :=
  p <- choose i32 true 0%i32 0%i32;
  let (z, choose_back) := p in
  z1 <- i32_add z 1%i32;
  if negb (z1 s= 1%i32)
  then Fail_ Failure
  else (
    p1 <- choose_back z1;
    let (x, y) := p1 in
    if negb (x s= 1%i32)
    then Fail_ Failure
    else if negb (y s= 0%i32) then Fail_ Failure else Ok tt)
.

(** Unit test for [paper::test_choose] *)
Check (test_choose )%return.

(** [paper::List]
    Source: 'tests/src/paper.rs', lines 38:0-38:16 *)
Inductive List_t (T : Type) :=
| List_Cons : T -> List_t T -> List_t T
| List_Nil : List_t T
.

Arguments List_Cons { _ }.
Arguments List_Nil { _ }.

(** [paper::list_nth_mut]:
    Source: 'tests/src/paper.rs', lines 45:0-45:67 *)
Fixpoint list_nth_mut
  (T : Type) (l : List_t T) (i : u32) :
  result (T * (T -> result (List_t T)))
  :=
  match l with
  | List_Cons x tl =>
    if i s= 0%u32
    then let back := fun (ret : T) => Ok (List_Cons ret tl) in Ok (x, back)
    else (
      i1 <- u32_sub i 1%u32;
      p <- list_nth_mut T tl i1;
      let (t, list_nth_mut_back) := p in
      let back :=
        fun (ret : T) => tl1 <- list_nth_mut_back ret; Ok (List_Cons x tl1) in
      Ok (t, back))
  | List_Nil => Fail_ Failure
  end
.

(** [paper::sum]:
    Source: 'tests/src/paper.rs', lines 60:0-60:32 *)
Fixpoint sum (l : List_t i32) : result i32 :=
  match l with
  | List_Cons x tl => i <- sum tl; i32_add x i
  | List_Nil => Ok 0%i32
  end
.

(** [paper::test_nth]:
    Source: 'tests/src/paper.rs', lines 71:0-71:17 *)
Definition test_nth : result unit :=
  let l := List_Cons 3%i32 List_Nil in
  let l1 := List_Cons 2%i32 l in
  p <- list_nth_mut i32 (List_Cons 1%i32 l1) 2%u32;
  let (x, list_nth_mut_back) := p in
  x1 <- i32_add x 1%i32;
  l2 <- list_nth_mut_back x1;
  i <- sum l2;
  if negb (i s= 7%i32) then Fail_ Failure else Ok tt
.

(** Unit test for [paper::test_nth] *)
Check (test_nth )%return.

(** [paper::call_choose]:
    Source: 'tests/src/paper.rs', lines 79:0-79:44 *)
Definition call_choose (p : (u32 * u32)) : result u32 :=
  let (px, py) := p in
  p1 <- choose u32 true px py;
  let (pz, choose_back) := p1 in
  pz1 <- u32_add pz 1%u32;
  p2 <- choose_back pz1;
  let (px1, _) := p2 in
  Ok px1
.

End Paper.