From a74f6b45d72834b5b8417297017bd81424123d98 Mon Sep 17 00:00:00 2001 From: xleroy Date: Sun, 7 Mar 2010 15:52:58 +0000 Subject: 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 --- backend/CSE.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'backend/CSE.v') diff --git a/backend/CSE.v b/backend/CSE.v index 98b7bbf5..ff79be54 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 -- cgit