aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/CSE2deps.v
diff options
context:
space:
mode:
Diffstat (limited to 'mppa_k1c/CSE2deps.v')
-rw-r--r--mppa_k1c/CSE2deps.v32
1 files changed, 0 insertions, 32 deletions
diff --git a/mppa_k1c/CSE2deps.v b/mppa_k1c/CSE2deps.v
deleted file mode 100644
index b4b80e2f..00000000
--- a/mppa_k1c/CSE2deps.v
+++ /dev/null
@@ -1,32 +0,0 @@
-(* *************************************************************)
-(* *)
-(* The Compcert verified compiler *)
-(* *)
-(* David Monniaux CNRS, VERIMAG *)
-(* *)
-(* Copyright VERIMAG. All rights reserved. *)
-(* This file is distributed under the terms of the INRIA *)
-(* Non-Commercial License Agreement. *)
-(* *)
-(* *************************************************************)
-
-Require Import BoolEqual Coqlib.
-Require Import AST Integers Floats.
-Require Import Values Memory Globalenvs Events.
-Require Import Op.
-
-
-Definition can_swap_accesses_ofs ofsr chunkr ofsw chunkw :=
- (0 <=? ofsw) && (ofsw <=? (Ptrofs.modulus - largest_size_chunk))
- && (0 <=? ofsr) && (ofsr <=? (Ptrofs.modulus - largest_size_chunk))
- && ((ofsw + size_chunk chunkw <=? ofsr) ||
- (ofsr + size_chunk chunkr <=? ofsw)).
-
-Definition may_overlap chunk addr args chunk' addr' args' :=
- match addr, addr', args, args' with
- | (Aindexed ofs), (Aindexed ofs'),
- (base :: nil), (base' :: nil) =>
- if peq base base'
- then negb (can_swap_accesses_ofs (Ptrofs.unsigned ofs') chunk' (Ptrofs.unsigned ofs) chunk)
- else true | _, _, _, _ => true
- end.