test(tests/lean/run/blast21): another blast test
This commit is contained in:
parent
3bd83b8e41
commit
093a212ed4
1 changed files with 19 additions and 0 deletions
19
tests/lean/run/blast21.lean
Normal file
19
tests/lean/run/blast21.lean
Normal file
|
@ -0,0 +1,19 @@
|
|||
namespace ex
|
||||
|
||||
constant typ : Type₁
|
||||
|
||||
constant subtype : typ → typ → Prop
|
||||
|
||||
constant subtype_refl : ∀ T, subtype T T
|
||||
|
||||
constant subtype_trans : ∀ S T U, subtype S T → subtype T U → subtype S U
|
||||
|
||||
attribute subtype_refl subtype_trans [backward]
|
||||
|
||||
lemma L1 : ∀ T1 T2 T3 T4 T5 T6, subtype T1 T2 → subtype T2 T3 → subtype T3 T4 → subtype T4 T5 → subtype T5 T6 → subtype T1 T6 :=
|
||||
by blast
|
||||
|
||||
reveal L1
|
||||
print L1
|
||||
|
||||
end ex
|
Loading…
Reference in a new issue