aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Integers.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-06-28 08:20:04 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-06-28 08:20:04 +0000
commita834a2aa0dfa9c2da663f5a645a6b086c0321871 (patch)
tree0104a7e5fa0a67155cef645a6adc8b8b147590c4 /lib/Integers.v
parentf0db487d8c8798b9899be03bf65bcb12524b9186 (diff)
downloadcompcert-kvx-a834a2aa0dfa9c2da663f5a645a6b086c0321871.tar.gz
compcert-kvx-a834a2aa0dfa9c2da663f5a645a6b086c0321871.zip
Merging the Princeton implementation of the memory model. Separate axioms in file lib/Axioms.v.
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1354 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'lib/Integers.v')
-rw-r--r--lib/Integers.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/lib/Integers.v b/lib/Integers.v
index f2aca962..f1440e9e 100644
--- a/lib/Integers.v
+++ b/lib/Integers.v
@@ -15,6 +15,7 @@
(** Formalizations of machine integers modulo $2^N$ #2<sup>N</sup>#. *)
+Require Import Axioms.
Require Import Coqlib.
(** * Comparisons *)
@@ -115,7 +116,7 @@ Lemma mkint_eq:
forall x y Px Py, x = y -> mkint x Px = mkint y Py.
Proof.
intros. subst y.
- generalize (proof_irrelevance _ Px Py); intro.
+ generalize (proof_irr Px Py); intro.
subst Py. reflexivity.
Qed.