aboutsummaryrefslogtreecommitdiffstats
path: root/backend/CSE3analysis.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/CSE3analysis.v')
-rw-r--r--backend/CSE3analysis.v12
1 files changed, 11 insertions, 1 deletions
diff --git a/backend/CSE3analysis.v b/backend/CSE3analysis.v
index 41fa67f6..456898cf 100644
--- a/backend/CSE3analysis.v
+++ b/backend/CSE3analysis.v
@@ -216,6 +216,16 @@ Section OPERATIONS.
else None
end
end.
-End OPERATIONS.
+
+ Definition oper2 (no : node) (dst : reg) (op: sym_op)(args : list reg)
+ (rel : RELATION.t) :=
+ let rel' := kill_reg dst rel in
+ match eq_find no {| eq_lhs := dst;
+ eq_op := op;
+ eq_args:= args |} with
+ | Some id => PSet.add id rel'
+ | None => rel'
+ end.
+ End OPERATIONS.
Definition totoro := RELATION.lub.