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
|
|
|
|
|
|
|
|
example : P :=
|
|
|
|
have H : P, from HP,
|
|
|
|
show P, by+ exact H
|
|
|
|
|
|
|
|
example : P :=
|
|
|
|
have H : P, from HP,
|
|
|
|
show P, begin+ exact H end
|
|
|
|
|
|
|
|
example : P :=
|
|
|
|
have H : P, from HP,
|
2016-02-29 19:28:20 +00:00
|
|
|
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
|