summaryrefslogtreecommitdiff
path: root/backend/CSE.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-03-07 15:52:58 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-03-07 15:52:58 +0000
commita74f6b45d72834b5b8417297017bd81424123d98 (patch)
treed291cf3f05397658f0fe9d8ecce9b8785a50d270 /backend/CSE.v
parent54cba6d4cae1538887f296a62be1c99378fe0916 (diff)
Merge of the newmem and newextcalls branches:
- Revised memory model with concrete representation of ints & floats, and per-byte access permissions - Revised Globalenvs implementation - Matching changes in all languages and proofs. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1282 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'backend/CSE.v')
-rw-r--r--backend/CSE.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/backend/CSE.v b/backend/CSE.v
index 98b7bbf..ff79be5 100644
--- a/backend/CSE.v
+++ b/backend/CSE.v
@@ -19,7 +19,7 @@ Require Import AST.
Require Import Integers.
Require Import Floats.
Require Import Values.
-Require Import Mem.
+Require Import Memory.
Require Import Globalenvs.
Require Import Op.
Require Import Registers.
@@ -265,7 +265,7 @@ Definition equation_holds
| Load chunk addr vl =>
exists a,
eval_addressing ge sp addr (List.map valuation vl) = Some a /\
- loadv chunk m a = Some (valuation vres)
+ Mem.loadv chunk m a = Some (valuation vres)
end.
Definition numbering_holds