lean2/tests/lean/run/830.lean

31 lines
405 B
Text
Raw Normal View History

2015-09-18 14:51:02 +00:00
variable P : Prop
premise HP : P
example : P :=
have H : P, from HP,
H
example : P :=
have H : P, from HP,
show P, from H
example : P :=
have H : P, from HP,
by exact H
2015-09-18 14:51:02 +00:00
example : P :=
have H : P, from HP,
show P, by exact H
2015-09-18 14:51:02 +00:00
example : P :=
have H : P, from HP,
show P, begin exact H end
2015-09-18 14:51:02 +00:00
example : P :=
have H : P, from HP,
show P, by exact H
2015-09-18 14:51:02 +00:00
example : P :=
assert H : P, from HP,
show P, by exact H