2015-09-18 07:51:02 -07: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,
|
2016-02-29 13:45:43 -08:00
|
|
|
by exact H
|
2015-09-18 07:51:02 -07:00
|
|
|
|
|
|
|
example : P :=
|
|
|
|
have H : P, from HP,
|
2016-02-29 13:45:43 -08:00
|
|
|
show P, by exact H
|
2015-09-18 07:51:02 -07:00
|
|
|
|
|
|
|
example : P :=
|
|
|
|
have H : P, from HP,
|
2016-02-29 13:45:43 -08:00
|
|
|
show P, begin exact H end
|
2015-09-18 07:51:02 -07:00
|
|
|
|
|
|
|
example : P :=
|
|
|
|
have H : P, from HP,
|
2016-02-29 11:28:20 -08:00
|
|
|
show P, by exact H
|
2015-09-18 07:51:02 -07:00
|
|
|
|
|
|
|
example : P :=
|
|
|
|
assert H : P, from HP,
|
|
|
|
show P, by exact H
|