lean2/tests/lean/gen_bug.lean
Leonardo de Moura b88b98ac22 feat(frontends/lean): try to add definition/theorem as axiom when it fails to be processed
The idea is to avoid a "tsunami" of error messages when a heavily used
theorem breaks in the beginning of the file
2015-03-13 14:47:21 -07:00

24 lines
425 B
Text

import logic
set_option pp.notation false
set_option pp.implicit true
theorem tst (A B : Type) (a : A) (b : B) : a == b → b == a :=
begin
intro H,
generalize B, -- Should produce an error
intro B',
apply (heq.symm H),
end
theorem tst2 (A B : Type) (a : A) (b : B) : a == b → b == a :=
begin
generalize a,
generalize b,
generalize B,
intro B',
intro b,
intro a,
intro H,
apply (heq.symm H),
end