2014-10-04 16:15:42 +00:00
|
|
|
import logic
|
|
|
|
open eq.ops
|
|
|
|
set_option pp.notation false
|
|
|
|
section
|
2014-10-09 14:13:06 +00:00
|
|
|
variable {A : Type}
|
|
|
|
variables {a b c d e : A}
|
2014-10-04 16:15:42 +00:00
|
|
|
theorem tst : a = b → b = c → c = d → d = e → a = e :=
|
|
|
|
take H1 H2 H3 H4,
|
|
|
|
have e1 : a = c,
|
|
|
|
proof
|
|
|
|
@eq.trans _ _ _ _ H1 H2
|
|
|
|
∎,
|
|
|
|
e1 ⬝ H3 ⬝ H4
|
|
|
|
end
|