lean2/tests/lean/run/676.lean

13 lines
184 B
Text
Raw Normal View History

import data.nat
open nat
inductive foo : Prop :=
mk : ∀ {a : nat}, a > 0 → foo
example (b : nat) (h : b > 1) : foo :=
begin
constructor,
exact b,
exact lt_of_succ_lt h
end