lean2/tests/lean/run/match_fun.lean

22 lines
441 B
Text

open bool nat
definition foo (b : bool) : nat → nat :=
match b with
| tt := λ x : nat, zero
| ff := λ y : nat, (succ zero)
end
example : foo tt 1 = zero := rfl
example : foo ff 1 = 1 := rfl
definition zero_fn := λ x : nat, zero
definition foo2 : bool → nat → nat
| foo2 tt := succ
| foo2 ff := zero_fn
example : foo2 tt 1 = 2 := rfl
example : foo2 tt 2 = 3 := rfl
example : foo2 ff 1 = 0 := rfl
example : foo2 ff 2 = 0 := rfl