aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/nsatz/Nsatz.v
diff options
context:
space:
mode:
Diffstat (limited to 'plugins/nsatz/Nsatz.v')
-rw-r--r--plugins/nsatz/Nsatz.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/nsatz/Nsatz.v b/plugins/nsatz/Nsatz.v
index 4f4f20396..5c1f4c470 100644
--- a/plugins/nsatz/Nsatz.v
+++ b/plugins/nsatz/Nsatz.v
@@ -241,7 +241,7 @@ Fixpoint interpret3 t fv {struct t}: R :=
| (PEpow t1 t2) =>
let v1 := interpret3 t1 fv in pow v1 (N.to_nat t2)
| (PEc t1) => (IZR1 t1)
- | (PEX n) => List.nth (pred (Pos.to_nat n)) fv 0
+ | (PEX _ n) => List.nth (pred (Pos.to_nat n)) fv 0
end.