aboutsummaryrefslogtreecommitdiffstats
path: root/src/bva
diff options
context:
space:
mode:
authorChantal Keller <Chantal.Keller@lri.fr>2020-07-06 12:44:56 +0200
committerChantal Keller <Chantal.Keller@lri.fr>2020-07-06 12:44:56 +0200
commit5d224b83ceda3d828ac446e3618bdd32cb23a00e (patch)
treef9baa7f7f7cc39c1f616cf7c46b20fca82d06bc5 /src/bva
parent9311585d0ce633e8e3b3a239c1d42d77219ef417 (diff)
parent6ddb77f5f60db1006c95552f893a71dd7571d966 (diff)
downloadsmtcoq-5d224b83ceda3d828ac446e3618bdd32cb23a00e.tar.gz
smtcoq-5d224b83ceda3d828ac446e3618bdd32cb23a00e.zip
Merge branch 'master' of github.com:smtcoq/smtcoq into coq-8.11
Diffstat (limited to 'src/bva')
-rw-r--r--src/bva/BVList.v6
-rw-r--r--src/bva/Bva_checker.v3
2 files changed, 4 insertions, 5 deletions
diff --git a/src/bva/BVList.v b/src/bva/BVList.v
index 6d64190..c9db26b 100644
--- a/src/bva/BVList.v
+++ b/src/bva/BVList.v
@@ -12,6 +12,7 @@
Require Import List Bool NArith Psatz Int63 Nnat ZArith.
Require Import Misc.
+Require Import ProofIrrelevance.
Import ListNotations.
Local Open Scope list_scope.
Local Open Scope N_scope.
@@ -21,9 +22,6 @@ Local Open Scope bool_scope.
Set Implicit Arguments.
Unset Strict Implicit.
-(* We temporarily assume proof irrelevance to handle dependently typed
- bit vectors *)
-Axiom proof_irrelevance : forall (P : Prop) (p1 p2 : P), p1 = p2.
Lemma inj a a' : N.to_nat a = N.to_nat a' -> a = a'.
Proof. intros. lia. Qed.
@@ -303,7 +301,7 @@ Module RAW2BITVECTOR (M:RAWBITVECTOR) <: BITVECTOR.
Proof.
unfold bv_eq. rewrite M.bv_eq_reflect. split.
- revert a b. intros [a Ha] [b Hb]. simpl. intros ->.
- rewrite (proof_irrelevance Ha Hb). reflexivity.
+ rewrite (proof_irrelevance _ Ha Hb). reflexivity.
- intros. case a in *. case b in *. simpl in *.
now inversion H. (* now intros ->. *)
Qed.
diff --git a/src/bva/Bva_checker.v b/src/bva/Bva_checker.v
index f066b54..c0fb520 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,