aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GiblePargenproofEquiv.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/GiblePargenproofEquiv.v')
-rw-r--r--src/hls/GiblePargenproofEquiv.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/src/hls/GiblePargenproofEquiv.v b/src/hls/GiblePargenproofEquiv.v
index 5f28d53..da2b2c1 100644
--- a/src/hls/GiblePargenproofEquiv.v
+++ b/src/hls/GiblePargenproofEquiv.v
@@ -1396,6 +1396,10 @@ Lemma check_mutexcl_correct:
predicated_mutexcl pe.
Proof. Admitted.
+Lemma check_mutexcl_singleton :
+ check_mutexcl (NE.singleton (T, EEbase)) = true.
+Proof. Admitted.
+
Definition check_mutexcl_tree {A} (f: PTree.t (predicated A)) :=
forall_ptree (fun _ => check_mutexcl) f.