aboutsummaryrefslogtreecommitdiffstats
path: root/backend/CSE3analysis.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-03-12 16:46:06 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-03-12 16:46:06 +0100
commitc6ebd73465ef895c6ea5e240f9c784463a6a0fe5 (patch)
tree15dec58036a4ddf49954cd25565b50e17bc1b292 /backend/CSE3analysis.v
parent9efb4d87c549087e2ef16103a6993a1f99328348 (diff)
downloadcompcert-kvx-c6ebd73465ef895c6ea5e240f9c784463a6a0fe5.tar.gz
compcert-kvx-c6ebd73465ef895c6ea5e240f9c784463a6a0fe5.zip
removed second analysis phase
Diffstat (limited to 'backend/CSE3analysis.v')
-rw-r--r--backend/CSE3analysis.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/backend/CSE3analysis.v b/backend/CSE3analysis.v
index 643b752a..69c21113 100644
--- a/backend/CSE3analysis.v
+++ b/backend/CSE3analysis.v
@@ -329,9 +329,11 @@ Definition apply_instr' (tenv : typing_env) code (pc : node) (ro : RB.t) : RB.t
end
end.
+Definition invariants := PMap.t RB.t.
+
Definition internal_analysis
(tenv : typing_env)
- (f : RTL.function) := DS.fixpoint
+ (f : RTL.function) : option invariants := DS.fixpoint
(RTL.fn_code f) RTL.successors_instr
(apply_instr' tenv (RTL.fn_code f)) (RTL.fn_entrypoint f) (Some RELATION.top).