lean2/tests/lean/subst2.lean.expected.out
Leonardo de Moura 88235d2922 feat(library/tactic/apply_tactic): try other solutions produced by the elaborator
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-12-25 11:51:27 -08:00

15 lines
577 B
Text

Set: pp::colors
Set: pp::unicode
Proved: T
Theorem T (A : Type) (p : A → Bool) (f : A → A → A) : ∀ x y z : A,
p (f x x) ⇒ x = y ⇒ x = z ⇒ p (f y z) :=
ForallIntro
(λ x : A,
ForallIntro
(λ x::1 : A,
ForallIntro
(λ x::2 : A,
Discharge
(λ H : p (f x x),
Discharge
(λ H::1 : x = x::1, Discharge (λ H::2 : x = x::2, Subst (Subst H H::1) H::2))))))