aboutsummaryrefslogtreecommitdiff
path: root/src/Nsatz.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Nsatz.v')
-rw-r--r--src/Nsatz.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/Nsatz.v b/src/Nsatz.v
index c8a648626..469ba4c29 100644
--- a/src/Nsatz.v
+++ b/src/Nsatz.v
@@ -1,5 +1,5 @@
(*** Tactics for manipulating polynomial equations *)
-Require Nsatz.
+Require Coq.nsatz.Nsatz.
Require Import List.
Generalizable All Variables.
@@ -109,6 +109,7 @@ Tactic Notation "nsatz" constr(n) :=
Tactic Notation "nsatz" := nsatz 1%nat || nsatz 2%nat || nsatz 3%nat || nsatz 4%nat || nsatz 5%nat.
Ltac nsatz_contradict :=
+ unfold not;
intros;
let domain := nsatz_guess_domain in
lazymatch type of domain with