You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
From Coq Require PeanoNat ZArith List Permutation Lia.
From AAC_tactics Require Import AAC.
From AAC_tactics Require Instances.
(** ** Introductory example
Here is a first example with relative numbers ([Z]): one can
rewrite an universally quantified hypothesis modulo the
associativity and commutativity of [Z.add]. *)
Section introduction.
Import ZArith.
Import Instances.Z.
Variables a b : Z.
Goal a + b = b + a.
aac_reflexivity.
Qed.
Goal forall c: bool, a + b = b + a.
intros c.
destruct c.
1,2: aac_reflexivity.
Fail Qed. (* The command has indeed failed with message: Some unresolved existential variables remain *)
Abort.
Goal forall c: bool, a + b = b + a.
intros c.
destruct c.
- aac_reflexivity.
- aac_reflexivity.
Qed.
End introduction.
The text was updated successfully, but these errors were encountered:
AAC tactics apparently don't handle goal selectors properly.
This might be an effect of #36.
Here is an example:
The text was updated successfully, but these errors were encountered: