summaryrefslogtreecommitdiff
path: root/tests/lean/misc-paper/Paper.lean
blob: 0b16fb8e372852892b1f26d1cf6c8d24efcf3e2f (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
122
123
-- THIS FILE WAS AUTOMATICALLY GENERATED BY AENEAS
-- [paper]
import Base.Primitives

/- [paper::ref_incr] -/
def ref_incr_fwd_back (x : I32) : Result I32 :=
  x + (I32.ofInt 1 (by intlit))

/- [paper::test_incr] -/
def test_incr_fwd : Result Unit :=
  do
    let x  ref_incr_fwd_back (I32.ofInt 0 (by intlit))
    if h: not (x = (I32.ofInt 1 (by intlit)))
    then Result.fail Error.panic
    else Result.ret ()

/- Unit test for [paper::test_incr] -/
#assert (test_incr_fwd == .ret ())

/- [paper::choose] -/
def choose_fwd (T : Type) (b : Bool) (x : T) (y : T) : Result T :=
  if h: b
  then Result.ret x
  else Result.ret y

/- [paper::choose] -/
def choose_back
  (T : Type) (b : Bool) (x : T) (y : T) (ret0 : T) : Result (T × T) :=
  if h: b
  then Result.ret (ret0, y)
  else Result.ret (x, ret0)

/- [paper::test_choose] -/
def test_choose_fwd : Result Unit :=
  do
    let z 
      choose_fwd I32 true (I32.ofInt 0 (by intlit)) (I32.ofInt 0 (by intlit))
    let z0  z + (I32.ofInt 1 (by intlit))
    if h: not (z0 = (I32.ofInt 1 (by intlit)))
    then Result.fail Error.panic
    else
      do
        let (x, y) 
          choose_back I32 true (I32.ofInt 0 (by intlit))
            (I32.ofInt 0 (by intlit)) z0
        if h: not (x = (I32.ofInt 1 (by intlit)))
        then Result.fail Error.panic
        else
          if h: not (y = (I32.ofInt 0 (by intlit)))
          then Result.fail Error.panic
          else Result.ret ()

/- Unit test for [paper::test_choose] -/
#assert (test_choose_fwd == .ret ())

/- [paper::List] -/
inductive list_t (T : Type) :=
| Cons : T -> list_t T -> list_t T
| Nil : list_t T

/- [paper::list_nth_mut] -/
def list_nth_mut_fwd (T : Type) (l : list_t T) (i : U32) : Result T :=
  match h: l with
  | list_t.Cons x tl =>
    if h: i = (U32.ofInt 0 (by intlit))
    then Result.ret x
    else do
           let i0  i - (U32.ofInt 1 (by intlit))
           list_nth_mut_fwd T tl i0
  | list_t.Nil => Result.fail Error.panic

/- [paper::list_nth_mut] -/
def list_nth_mut_back
  (T : Type) (l : list_t T) (i : U32) (ret0 : T) : Result (list_t T) :=
  match h: l with
  | list_t.Cons x tl =>
    if h: i = (U32.ofInt 0 (by intlit))
    then Result.ret (list_t.Cons ret0 tl)
    else
      do
        let i0  i - (U32.ofInt 1 (by intlit))
        let tl0  list_nth_mut_back T tl i0 ret0
        Result.ret (list_t.Cons x tl0)
  | list_t.Nil => Result.fail Error.panic

/- [paper::sum] -/
def sum_fwd (l : list_t I32) : Result I32 :=
  match h: l with
  | list_t.Cons x tl => do
                          let i  sum_fwd tl
                          x + i
  | list_t.Nil => Result.ret (I32.ofInt 0 (by intlit))

/- [paper::test_nth] -/
def test_nth_fwd : Result Unit :=
  do
    let l := list_t.Nil
    let l0 := list_t.Cons (I32.ofInt 3 (by intlit)) l
    let l1 := list_t.Cons (I32.ofInt 2 (by intlit)) l0
    let x 
      list_nth_mut_fwd I32 (list_t.Cons (I32.ofInt 1 (by intlit)) l1)
        (U32.ofInt 2 (by intlit))
    let x0  x + (I32.ofInt 1 (by intlit))
    let l2 
      list_nth_mut_back I32 (list_t.Cons (I32.ofInt 1 (by intlit)) l1)
        (U32.ofInt 2 (by intlit)) x0
    let i  sum_fwd l2
    if h: not (i = (I32.ofInt 7 (by intlit)))
    then Result.fail Error.panic
    else Result.ret ()

/- Unit test for [paper::test_nth] -/
#assert (test_nth_fwd == .ret ())

/- [paper::call_choose] -/
def call_choose_fwd (p : (U32 × U32)) : Result U32 :=
  do
    let (px, py) := p
    let pz  choose_fwd U32 true px py
    let pz0  pz + (U32.ofInt 1 (by intlit))
    let (px0, _)  choose_back U32 true px py pz0
    Result.ret px0