aboutsummaryrefslogtreecommitdiffstats
path: root/common/Memory.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-09-05 11:19:22 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-09-05 11:19:22 +0200
commitc4cc75dc6abcb0eee6f3288e96fea4aec540fd68 (patch)
treee63d0437c3f3cb43eb26cced8ad94acc62e82dad /common/Memory.v
parent7042070a3668ae149ec6a490b8e7c1a6aa82d6fe (diff)
downloadcompcert-kvx-c4cc75dc6abcb0eee6f3288e96fea4aec540fd68.tar.gz
compcert-kvx-c4cc75dc6abcb0eee6f3288e96fea4aec540fd68.zip
more proofs going through
Diffstat (limited to 'common/Memory.v')
-rw-r--r--common/Memory.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/common/Memory.v b/common/Memory.v
index b68a5049..cfd13601 100644
--- a/common/Memory.v
+++ b/common/Memory.v
@@ -39,6 +39,9 @@ Require Import Values.
Require Export Memdata.
Require Export Memtype.
+Definition default_notrap_load_value (chunk : memory_chunk) := Vundef.
+
+
(* To avoid useless definitions of inductors in extracted code. *)
Local Unset Elimination Schemes.
Local Unset Case Analysis Schemes.