Skip to content

Commit

Permalink
Removed not_symmetry from stdpp_tactics.v, importing not_symmetry fro…
Browse files Browse the repository at this point in the history
…m MathClasses.misc.util
  • Loading branch information
ndcroos committed Jul 30, 2024
1 parent 99feb0c commit b4d9a0e
Showing 1 changed file with 2 additions and 3 deletions.
5 changes: 2 additions & 3 deletions stdpp/stdpp_tactics.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,7 @@
Require Import

Check failure on line 1 in stdpp/stdpp_tactics.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:8.19)

Cannot find a physical path bound to logical path

Check failure on line 1 in stdpp/stdpp_tactics.v

View workflow job for this annotation

GitHub Actions / build (coqorg/coq:8.18)

Cannot find a physical path bound to logical path
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.

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
Expand Down

0 comments on commit b4d9a0e

Please sign in to comment.