lean2/tests/lean/pstate.lean

5 lines
114 B
Text
Raw Normal View History

import logic
theorem foo {A : Type} (a b c : A) : a = b → b = c → a = c :=
assume h₁ h₂, eq.trans h₁ _