summaryrefslogtreecommitdiff
path: root/lib/Integers.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-09 17:28:10 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-09 17:28:10 +0000
commite29b0c71f446ea6267711c7cc19294fd93fb81ad (patch)
tree0317ddbba0cc4a81175f6e05e337d56211a29a26 /lib/Integers.v
parent20eea14b1c678722642da5c22afd6e87b6cdf686 (diff)
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 'lib/Integers.v')
-rw-r--r--lib/Integers.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/lib/Integers.v b/lib/Integers.v
index 0575436..2c74e80 100644
--- a/lib/Integers.v
+++ b/lib/Integers.v
@@ -57,6 +57,10 @@ Module Type WORDSIZE.
Axiom wordsize_not_zero: wordsize <> 0%nat.
End WORDSIZE.
+(* To avoid useless definitions of inductors in extracted code. *)
+Local Unset Elimination Schemes.
+Local Unset Case Analysis Schemes.
+
Module Make(WS: WORDSIZE).
Definition wordsize: nat := WS.wordsize.