aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Locations.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Locations.v')
-rw-r--r--backend/Locations.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/backend/Locations.v b/backend/Locations.v
index 1270e1d3..8a0b5ea2 100644
--- a/backend/Locations.v
+++ b/backend/Locations.v
@@ -280,6 +280,15 @@ Module Loc.
apply overlap_aux_false_1. exact H0.
Qed.
+ Definition diff_dec (l1 l2: loc) : { Loc.diff l1 l2 } + {~Loc.diff l1 l2}.
+ Proof.
+ intros. case (eq l1 l2); intros.
+ right. rewrite e. apply same_not_diff.
+ case_eq (overlap l1 l2); intros.
+ right. apply overlap_not_diff; auto.
+ left. apply non_overlap_diff; auto.
+ Qed.
+
(** We now redefine some standard notions over lists, using the [Loc.diff]
predicate instead of standard disequality [<>].