a4c0699e81
See issue #676 Add new test demonstrating why it is useful to have the old semantics for 'constructor'
12 lines
185 B
Text
12 lines
185 B
Text
import data.nat
|
|
open nat
|
|
|
|
inductive foo : Prop :=
|
|
mk : ∀ {a : nat}, a > 0 → foo
|
|
|
|
example (b : nat) (h : b > 1) : foo :=
|
|
begin
|
|
fconstructor,
|
|
exact b,
|
|
exact lt_of_succ_lt h
|
|
end
|