From a834a2aa0dfa9c2da663f5a645a6b086c0321871 Mon Sep 17 00:00:00 2001 From: xleroy Date: Mon, 28 Jun 2010 08:20:04 +0000 Subject: 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 --- lib/Parmov.v | 7 ++++--- 1 file changed, 4 insertions(+), 3 deletions(-) (limited to 'lib/Parmov.v') 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 -- cgit