2014-08-24 19:58:48 -07:00
|
|
|
import data.num
|
2014-09-04 16:36:06 -07:00
|
|
|
|
2014-07-15 01:19:47 +01:00
|
|
|
|
|
|
|
namespace foo
|
2014-10-02 16:20:52 -07:00
|
|
|
constant le : num → num → Prop
|
2014-07-15 01:19:47 +01:00
|
|
|
axiom le_trans {a b c : num} : le a b → le b c → le a c
|
2015-05-02 15:15:35 -07:00
|
|
|
attribute le_trans [trans]
|
2014-10-21 15:27:45 -07:00
|
|
|
infix `≤` := le
|
2014-08-07 16:59:08 -07:00
|
|
|
end foo
|
2014-07-15 01:19:47 +01:00
|
|
|
|
|
|
|
namespace foo
|
|
|
|
theorem T {a b c d : num} : a ≤ b → b ≤ c → c ≤ d → a ≤ d
|
|
|
|
:= assume H1 H2 H3,
|
|
|
|
calc a ≤ b : H1
|
|
|
|
... ≤ c : H2
|
|
|
|
... ≤ d : H3
|
2014-08-07 16:59:08 -07:00
|
|
|
end foo
|