Skip to content

Commit

Permalink
removed 'easy' to 'done' replacements
Browse files Browse the repository at this point in the history
  • Loading branch information
ndcroos committed Jul 31, 2024
1 parent 2a8e123 commit 6fac6fe
Showing 1 changed file with 36 additions and 0 deletions.
36 changes: 36 additions & 0 deletions misc/stdpp_tactics.v
Original file line number Diff line number Diff line change
@@ -0,0 +1,36 @@
From Coq Require Export RelationClasses Relation_Definitions Lia.

Module FastDoneTactic.

Lemma not_symmetry {A} `{R : relation A, !Symmetric R} x y : ~ R x y -> ~ R y x.
Proof. intuition. Qed.

Ltac fast_done :=
solve
[ eassumption
| symmetry; eassumption
| apply not_symmetry; eassumption
| reflexivity ].
Tactic Notation "fast_by" tactic(tac) :=
tac; fast_done.

End FastDoneTactic.

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 ]
].

0 comments on commit 6fac6fe

Please sign in to comment.