lean2/tests/lean/run/676.lean
Leonardo de Moura a4c0699e81 feat(library/tactic/constructor_tactic): restore 'constructor' tactic old semantics, add 'fconstructor' tactic
See issue #676

Add new test demonstrating why it is useful to have the old semantics
for 'constructor'
2015-06-17 23:48:54 -07:00

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