Skip to content
Snippets Groups Projects
Commit c17ab51c authored by Ralf Jung's avatar Ralf Jung
Browse files

coqdoc

parent 14ccc4c8
No related branches found
No related tags found
1 merge request!261add tactic for solving computable goals
...@@ -136,12 +136,12 @@ Lemma bool_decide_eq_false_2 P `{!Decision P}: ¬P → bool_decide P = false. ...@@ -136,12 +136,12 @@ Lemma bool_decide_eq_false_2 P `{!Decision P}: ¬P → bool_decide P = false.
Proof. apply bool_decide_eq_false. Qed. Proof. apply bool_decide_eq_false. Qed.
(** The tactic [compute_done] solves the following kinds of goals: (** The tactic [compute_done] solves the following kinds of goals:
- Goals `P` where `Decidable P` can be derived. - Goals [P] where [Decidable P] can be derived.
- Goals that compute to `True` or `x = x`. - Goals that compute to [True] or [x = x].
The goal must be a ground term for this, i.e., not contain variables (that do The goal must be a ground term for this, i.e., not contain variables (that do
not compute away). The goal is solved by using `vm_compute` and then using a not compute away). The goal is solved by using [vm_compute] and then using a
trivial proof term (`I`/`eq_refl`). *) trivial proof term ([I]/[eq_refl]). *)
Tactic Notation "compute_done" := Tactic Notation "compute_done" :=
try apply (bool_decide_unpack _); try apply (bool_decide_unpack _);
vm_compute; vm_compute;
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment