aboutsummaryrefslogtreecommitdiffstats
path: root/src/bva/Bva_checker.v
diff options
context:
space:
mode:
authorChantal Keller <Chantal.Keller@lri.fr>2020-07-01 10:29:37 +0200
committerChantal Keller <Chantal.Keller@lri.fr>2020-07-01 10:29:37 +0200
commit6a0a78282219d1402457222d5728286836ab9f0f (patch)
treed40d0dc859a2fc7c3272dd8b540c5d8115fd7563 /src/bva/Bva_checker.v
parent7a465031fb18e4af2c90c04b435ed336bbdb79a3 (diff)
downloadsmtcoq-6a0a78282219d1402457222d5728286836ab9f0f.tar.gz
smtcoq-6a0a78282219d1402457222d5728286836ab9f0f.zip
Use officiel library for proof irrelevance
Diffstat (limited to 'src/bva/Bva_checker.v')
-rw-r--r--src/bva/Bva_checker.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/src/bva/Bva_checker.v b/src/bva/Bva_checker.v
index eebf5f9..20cc2cf 100644
--- a/src/bva/Bva_checker.v
+++ b/src/bva/Bva_checker.v
@@ -19,6 +19,7 @@ Require Import Int63 Int63Properties PArray SMT_classes ZArith.
Require Import Misc State SMT_terms BVList Psatz.
Require Import Bool List BoolEq NZParity Nnat.
Require Import BinPos BinNat Pnat Init.Peano.
+Require Import ProofIrrelevance.
Require FArray.
@@ -1474,7 +1475,7 @@ Proof. intros. destruct a, b.
unfold BITVECTOR_LIST.bv in H.
revert wf0.
rewrite H. intros.
- now rewrite (proof_irrelevance wf0 wf1).
+ now rewrite (proof_irrelevance _ wf0 wf1).
Qed.
Lemma nth_eq0: forall i a b xs ys,