lean2/tests/lean/subst3.lean.expected.out
Leonardo de Moura a3dde29f3c feat(frontends/lua/parser): allow users to specify the precedence of macros
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-12-25 12:27:56 -08:00

14 lines
523 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
(λ y : A,
ForallIntro
(λ z : A,
Discharge
(λ H1 : p (f x x),
Discharge (λ H2 : x = y, Discharge (λ H3 : x = z, Subst (Subst H1 H2) H3))))))