diff options
Diffstat (limited to 'tests/lean/Paper.lean')
-rw-r--r-- | tests/lean/Paper.lean | 57 |
1 files changed, 29 insertions, 28 deletions
diff --git a/tests/lean/Paper.lean b/tests/lean/Paper.lean index 9f63b460..ade65656 100644 --- a/tests/lean/Paper.lean +++ b/tests/lean/Paper.lean @@ -4,39 +4,40 @@ import Base open Primitives namespace paper -/- [paper::ref_incr] -/ -def ref_incr_fwd_back (x : I32) : Result I32 := +/- [paper::ref_incr]: merged forward/backward function + (there is a single backward function, and the forward function returns ()) -/ +def ref_incr (x : I32) : Result I32 := x + (I32.ofInt 1 (by intlit)) -/- [paper::test_incr] -/ -def test_incr_fwd : Result Unit := +/- [paper::test_incr]: forward function -/ +def test_incr : Result Unit := do - let x ← ref_incr_fwd_back (I32.ofInt 0 (by intlit)) + let x ← ref_incr (I32.ofInt 0 (by intlit)) if 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 ()) +#assert (test_incr == .ret ()) -/- [paper::choose] -/ -def choose_fwd (T : Type) (b : Bool) (x : T) (y : T) : Result T := +/- [paper::choose]: forward function -/ +def choose (T : Type) (b : Bool) (x : T) (y : T) : Result T := if b then Result.ret x else Result.ret y -/- [paper::choose] -/ +/- [paper::choose]: backward function 0 -/ def choose_back (T : Type) (b : Bool) (x : T) (y : T) (ret0 : T) : Result (T × T) := if b then Result.ret (ret0, y) else Result.ret (x, ret0) -/- [paper::test_choose] -/ -def test_choose_fwd : Result Unit := +/- [paper::test_choose]: forward function -/ +def test_choose : Result Unit := do let z ← - choose_fwd I32 true (I32.ofInt 0 (by intlit)) (I32.ofInt 0 (by intlit)) + choose I32 true (I32.ofInt 0 (by intlit)) (I32.ofInt 0 (by intlit)) let z0 ← z + (I32.ofInt 1 (by intlit)) if not (z0 = (I32.ofInt 1 (by intlit))) then Result.fail Error.panic @@ -53,25 +54,25 @@ def test_choose_fwd : Result Unit := else Result.ret () /- Unit test for [paper::test_choose] -/ -#assert (test_choose_fwd == .ret ()) +#assert (test_choose == .ret ()) /- [paper::List] -/ inductive List (T : Type) := | Cons : T → List T → List T | Nil : List T -/- [paper::list_nth_mut] -/ -divergent def list_nth_mut_fwd (T : Type) (l : List T) (i : U32) : Result T := +/- [paper::list_nth_mut]: forward function -/ +divergent def list_nth_mut (T : Type) (l : List T) (i : U32) : Result T := match l with | List.Cons x tl => if 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_nth_mut T tl i0 | List.Nil => Result.fail Error.panic -/- [paper::list_nth_mut] -/ +/- [paper::list_nth_mut]: backward function 0 -/ divergent def list_nth_mut_back (T : Type) (l : List T) (i : U32) (ret0 : T) : Result (List T) := match l with @@ -85,40 +86,40 @@ divergent def list_nth_mut_back Result.ret (List.Cons x tl0) | List.Nil => Result.fail Error.panic -/- [paper::sum] -/ -divergent def sum_fwd (l : List I32) : Result I32 := +/- [paper::sum]: forward function -/ +divergent def sum (l : List I32) : Result I32 := match l with | List.Cons x tl => do - let i ← sum_fwd tl + let i ← sum tl x + i | List.Nil => Result.ret (I32.ofInt 0 (by intlit)) -/- [paper::test_nth] -/ -def test_nth_fwd : Result Unit := +/- [paper::test_nth]: forward function -/ +def test_nth : Result Unit := do let l := List.Nil let l0 := List.Cons (I32.ofInt 3 (by intlit)) l let l1 := List.Cons (I32.ofInt 2 (by intlit)) l0 let x ← - list_nth_mut_fwd I32 (List.Cons (I32.ofInt 1 (by intlit)) l1) + list_nth_mut I32 (List.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.Cons (I32.ofInt 1 (by intlit)) l1) (U32.ofInt 2 (by intlit)) x0 - let i ← sum_fwd l2 + let i ← sum l2 if 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 ()) +#assert (test_nth == .ret ()) -/- [paper::call_choose] -/ -def call_choose_fwd (p : (U32 × U32)) : Result U32 := +/- [paper::call_choose]: forward function -/ +def call_choose (p : (U32 × U32)) : Result U32 := do let (px, py) := p - let pz ← choose_fwd U32 true px py + let pz ← choose U32 true px py let pz0 ← pz + (U32.ofInt 1 (by intlit)) let (px0, _) ← choose_back U32 true px py pz0 Result.ret px0 |