lean2/tests/lean/bug1.lean.expected.out
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

19 lines
713 B
Text

bug1.lean:9:7: error: type mismatch at definition 'and_intro1', has type
∀ (p q : bool),
p → q → (∀ (c : bool), (p → q → c) → c)
but is expected to have type
∀ (p q : bool),
p → q → a
bug1.lean:13:7: error: type mismatch at definition 'and_intro2', has type
∀ (p q : bool),
p → q → (∀ (c : bool), (p → q → c) → c)
but is expected to have type
∀ (p q : bool),
p → q → p ∧ p
bug1.lean:17:7: error: type mismatch at definition 'and_intro3', has type
∀ (p q : bool),
p → q → (∀ (c : bool), (p → q → c) → c)
but is expected to have type
∀ (p q : bool),
p → q → q ∧ p
and_intro4 : ∀ (p q : bool), p → q → p ∧ q