lean2/tests/lean/abst.lean.expected.out

10 lines
334 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Imported 'int'
Assumed: PlusComm
Assumed: a
Abst (λ x : , PlusComm a x) : (λ x : , a + x) == (λ x : , x + a)
Set: lean::pp::implicit
@Abst (λ x : , ) (λ x : , a + x) (λ x : , x + a) (λ x : , PlusComm a x) :
(λ x : , a + x) == (λ x : , x + a)