aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/abstractbb/DepTreeTheory.v
diff options
context:
space:
mode:
Diffstat (limited to 'mppa_k1c/abstractbb/DepTreeTheory.v')
-rw-r--r--mppa_k1c/abstractbb/DepTreeTheory.v10
1 files changed, 4 insertions, 6 deletions
diff --git a/mppa_k1c/abstractbb/DepTreeTheory.v b/mppa_k1c/abstractbb/DepTreeTheory.v
index 6f017378..353e9160 100644
--- a/mppa_k1c/abstractbb/DepTreeTheory.v
+++ b/mppa_k1c/abstractbb/DepTreeTheory.v
@@ -129,19 +129,17 @@ with list_exp_tree (le: list_exp) (d old: deps): list_tree :=
Definition failsafe (t: tree): bool :=
match t with
| Tname x => true
- | Top o Tnil =>
- match op_eval ge o nil with
- | Some _ => true
- | None => false
- end
+ | Top o Tnil => is_constant o
| _ => false
end.
+Local Hint Resolve is_constant_correct.
+
Lemma failsafe_correct (t: tree) m: failsafe t = true -> tree_eval t m <> None.
Proof.
destruct t; simpl; try congruence.
destruct l; simpl; try congruence.
- destruct (op_eval ge o nil); try congruence.
+ eauto.
Qed.
Fixpoint macro_deps (i: macro) (d old: deps): deps :=