aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Parmov.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/Parmov.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/Parmov.v')
-rw-r--r--lib/Parmov.v7
1 files changed, 4 insertions, 3 deletions
diff --git a/lib/Parmov.v b/lib/Parmov.v
index edb267e4..493b0bdd 100644
--- a/lib/Parmov.v
+++ b/lib/Parmov.v
@@ -2,8 +2,8 @@
(* *)
(* The Compcert verified compiler *)
(* *)
-(* Laurence Rideau, INRIA Sophia-Antipolis-Méditerranée *)
-(* Bernard Paul Serpette, INRIA Sophia-Antipolis-Méditerranée *)
+(* Laurence Rideau, INRIA Sophia-Antipolis-M\u00e9diterran\u00e9e *)
+(* Bernard Paul Serpette, INRIA Sophia-Antipolis-M\u00e9diterran\u00e9e *)
(* Xavier Leroy, INRIA Paris-Rocquencourt *)
(* *)
(* Copyright Institut National de Recherche en Informatique et en *)
@@ -53,6 +53,7 @@
*)
Require Import Relations.
+Require Import Axioms.
Require Import Coqlib.
Require Recdef.
@@ -99,7 +100,7 @@ Definition env := reg -> val.
Lemma env_ext:
forall (e1 e2: env),
(forall r, e1 r = e2 r) -> e1 = e2.
-Proof (extensionality reg val).
+Proof (@extensionality reg val).
(** The main operation over environments is update: it assigns
a value [v] to a register [r] and preserves the values of other