summaryrefslogtreecommitdiff
path: root/tests/coq/misc/Paper.v
blob: 175a523d4dbed4aa574a57b625eb49510f5f41e2 (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]: merged forward/backward function
    (there is a single backward function, and the forward function returns ()) *)
Definition ref_incr_fwd_back (x : i32) : result i32 :=
  i32_add x 1%i32.

(** [paper::test_incr]: forward function *)
Definition test_incr_fwd : result unit :=
  x <- ref_incr_fwd_back 0%i32;
  if negb (x s= 1%i32) then Fail_ Failure else Return tt
.

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

(** [paper::choose]: forward function *)
Definition choose_fwd (T : Type) (b : bool) (x : T) (y : T) : result T :=
  if b then Return x else Return y
.

(** [paper::choose]: backward function 0 *)
Definition choose_back
  (T : Type) (b : bool) (x : T) (y : T) (ret : T) : result (T * T) :=
  if b then Return (ret, y) else Return (x, ret)
.

(** [paper::test_choose]: forward function *)
Definition test_choose_fwd : result unit :=
  z <- choose_fwd i32 true 0%i32 0%i32;
  z0 <- i32_add z 1%i32;
  if negb (z0 s= 1%i32)
  then Fail_ Failure
  else (
    p <- choose_back i32 true 0%i32 0%i32 z0;
    let (x, y) := p in
    if negb (x s= 1%i32)
    then Fail_ Failure
    else if negb (y s= 0%i32) then Fail_ Failure else Return tt)
.

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

(** [paper::List] *)
Inductive List_t (T : Type) :=
| ListCons : T -> List_t T -> List_t T
| ListNil : List_t T
.

Arguments ListCons {T} _ _.
Arguments ListNil {T}.

(** [paper::list_nth_mut]: forward function *)
Fixpoint list_nth_mut_fwd (T : Type) (l : List_t T) (i : u32) : result T :=
  match l with
  | ListCons x tl =>
    if i s= 0%u32
    then Return x
    else (i0 <- u32_sub i 1%u32; list_nth_mut_fwd T tl i0)
  | ListNil => Fail_ Failure
  end
.

(** [paper::list_nth_mut]: backward function 0 *)
Fixpoint list_nth_mut_back
  (T : Type) (l : List_t T) (i : u32) (ret : T) : result (List_t T) :=
  match l with
  | ListCons x tl =>
    if i s= 0%u32
    then Return (ListCons ret tl)
    else (
      i0 <- u32_sub i 1%u32;
      tl0 <- list_nth_mut_back T tl i0 ret;
      Return (ListCons x tl0))
  | ListNil => Fail_ Failure
  end
.

(** [paper::sum]: forward function *)
Fixpoint sum_fwd (l : List_t i32) : result i32 :=
  match l with
  | ListCons x tl => i <- sum_fwd tl; i32_add x i
  | ListNil => Return 0%i32
  end
.

(** [paper::test_nth]: forward function *)
Definition test_nth_fwd : result unit :=
  let l := ListNil in
  let l0 := ListCons 3%i32 l in
  let l1 := ListCons 2%i32 l0 in
  x <- list_nth_mut_fwd i32 (ListCons 1%i32 l1) 2%u32;
  x0 <- i32_add x 1%i32;
  l2 <- list_nth_mut_back i32 (ListCons 1%i32 l1) 2%u32 x0;
  i <- sum_fwd l2;
  if negb (i s= 7%i32) then Fail_ Failure else Return tt
.

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

(** [paper::call_choose]: forward function *)
Definition call_choose_fwd (p : (u32 * u32)) : result u32 :=
  let (px, py) := p in
  pz <- choose_fwd u32 true px py;
  pz0 <- u32_add pz 1%u32;
  p0 <- choose_back u32 true px py pz0;
  let (px0, _) := p0 in
  Return px0
.

End Paper .