aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GiblePargenproofEquiv.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2023-05-12 18:36:34 +0100
committerYann Herklotz <git@yannherklotz.com>2023-05-12 18:36:34 +0100
commit17f479648a2912e6a7c8c20664645f22a75cf1b8 (patch)
tree26155bea69eb46b37856d5f66158045afc1cf3f5 /src/hls/GiblePargenproofEquiv.v
parentc1778dc2f1a5de755b32f8c4655a718c109c6489 (diff)
downloadvericert-17f479648a2912e6a7c8c20664645f22a75cf1b8.tar.gz
vericert-17f479648a2912e6a7c8c20664645f22a75cf1b8.zip
Rename backwards proof
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.