Set: pp::colors Set: pp::unicode Imported 'macros' 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) := forall::intro (λ x : A, forall::intro (λ y : A, forall::intro (λ z : A, discharge (λ H1 : p (f x x), discharge (λ H2 : x = y, discharge (λ H3 : x = z, subst (subst H1 H2) H3))))))