lean2/tests/lean/sum3.lean.expected.out
Leonardo de Moura 1ec01f5757 refactor(builtin): merge pair.lean with kernel.lean, and add basic theorems
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-02-07 16:04:44 -08:00

29 lines
675 B
Text
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

Set: pp::colors
Set: pp::unicode
Imported 'macros'
Imported 'subtype'
Imported 'optional'
Using: subtype
Using: optional
Defined: sum_pred
Defined: sum
Proved: sum::inl_pred
Proved: sum::inr_pred
Proved: sum::inhabl
Proved: sum::inhabr
Defined: sum::inl
Defined: sum::inr
Proved: sum::inl_inj
Proved: sum::inr_inj
Proved: sum::distinct
sum3.lean:96:0: error: invalid tactic command, unexpected end of file
Proof state:
A :
(Type U),
B :
(Type U),
n :
sum A B,
pred :
(proj1 (subtype::rep n) = optional::none) ≠ (proj2 (subtype::rep n) = optional::none)
⊢ (∃ a : A, n = sum::inl a B) (∃ b : B, n = sum::inr A b)