lean2/tests/lean/run/measurable.lean

8 lines
207 B
Text
Raw Normal View History

open prod nat
example (a b : nat) : size_of (a, true, bool.tt, (λ c d : nat, c + d), option.some b) = a + b :=
rfl
example : size_of (pair (pair (pair 2 true) (λ a : nat, a)) (option.some 3)) = 5 :=
rfl