aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/omega/PreOmega.v
diff options
context:
space:
mode:
Diffstat (limited to 'contrib/omega/PreOmega.v')
-rw-r--r--contrib/omega/PreOmega.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/contrib/omega/PreOmega.v b/contrib/omega/PreOmega.v
index 0a4328497..47e22a97f 100644
--- a/contrib/omega/PreOmega.v
+++ b/contrib/omega/PreOmega.v
@@ -412,12 +412,12 @@ Ltac zify_N_op :=
| |- context [ Z_of_N (Nsucc ?a) ] => rewrite (Z_of_N_succ a)
(* Nmult -> Zmult and a positivity hypothesis *)
- | H : context [ Z_of_N (Pmult ?a ?b) ] |- _ =>
+ | H : context [ Z_of_N (Nmult ?a ?b) ] |- _ =>
let H:= fresh "H" in
- assert (H:=Z_of_N_le_0 (Pmult a b)); rewrite (Z_of_N_mult a b) in *
- | |- context [ Z_of_N (Pmult ?a ?b) ] =>
+ assert (H:=Z_of_N_le_0 (Nmult a b)); rewrite (Z_of_N_mult a b) in *
+ | |- context [ Z_of_N (Nmult ?a ?b) ] =>
let H:= fresh "H" in
- assert (H:=Z_of_N_le_0 (Pmult a b)); rewrite (Z_of_N_mult a b) in *
+ assert (H:=Z_of_N_le_0 (Nmult a b)); rewrite (Z_of_N_mult a b) in *
(* atoms of type N : we add a positivity condition (if not already there) *)
| H : context [ Z_of_N ?a ] |- _ =>