Skip to content

Commit

Permalink
Hide fast_done tactic
Browse files Browse the repository at this point in the history
  • Loading branch information
ndcroos committed Jul 30, 2024
1 parent b4d9a0e commit cd217a1
Showing 1 changed file with 24 additions and 15 deletions.
39 changes: 24 additions & 15 deletions stdpp/stdpp_tactics.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,8 @@ Require Import
MathClasses.misc.util.

Check failure on line 2 in stdpp/stdpp_tactics.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:dev)

Cannot find a physical path bound to logical path
From Coq Require Export RelationClasses Relation_Definitions Lia.

Module FastDoneTactic.

Ltac fast_done :=
solve
[ eassumption
Expand All @@ -11,18 +13,25 @@ Ltac fast_done :=
Tactic Notation "fast_by" tactic(tac) :=
tac; fast_done.

Ltac done :=
solve
[ repeat first
[ fast_done
| solve [trivial]
(* All the tactics below will introduce themselves anyway, or make no sense
for goals of product type. So this is a good place for us to do it. *)
| progress intros
| solve [symmetry; trivial]
| solve [apply not_symmetry; trivial]
| discriminate
| contradiction
| split
| match goal with H : ~ _ |- _ => case H; clear H; fast_done end ]
].
End FastDoneTactic.

Section DoneSection.
Import FastDoneTactic.

Ltac done :=
solve
[ repeat first
[ fast_done
| solve [trivial]
(* All the tactics below will introduce themselves anyway, or make no sense
for goals of product type. So this is a good place for us to do it. *)
| progress intros
| solve [symmetry; trivial]
| solve [apply not_symmetry; trivial]
| discriminate
| contradiction
| split
| match goal with H : ~ _ |- _ => case H; clear H; fast_done end ]
].

End DoneSection.

0 comments on commit cd217a1

Please sign in to comment.