aboutsummaryrefslogtreecommitdiffstats
path: root/common/Memory.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-09 17:28:10 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-09 17:28:10 +0000
commite29b0c71f446ea6267711c7cc19294fd93fb81ad (patch)
tree0317ddbba0cc4a81175f6e05e337d56211a29a26 /common/Memory.v
parent20eea14b1c678722642da5c22afd6e87b6cdf686 (diff)
downloadcompcert-kvx-e29b0c71f446ea6267711c7cc19294fd93fb81ad.tar.gz
compcert-kvx-e29b0c71f446ea6267711c7cc19294fd93fb81ad.zip
Assorted cleanups, esp. to avoid generating _rec and _rect recursors in
submodules. (Extraction does not remove them, then.) common/Switch: replaced use of FMaps by our own Maps. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2139 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'common/Memory.v')
-rw-r--r--common/Memory.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/common/Memory.v b/common/Memory.v
index 04a3dda6..bfaf67d1 100644
--- a/common/Memory.v
+++ b/common/Memory.v
@@ -36,6 +36,10 @@ Require Import Values.
Require Export Memdata.
Require Export Memtype.
+(* To avoid useless definitions of inductors in extracted code. *)
+Local Unset Elimination Schemes.
+Local Unset Case Analysis Schemes.
+
Local Notation "a # b" := (ZMap.get b a) (at level 1).
Module Mem <: MEM.