aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/Abstr.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-06-03 18:08:05 +0100
committerYann Herklotz <git@yannherklotz.com>2022-06-03 18:08:05 +0100
commitdb4da00aea8b51bc9d90d83f981b9163eec3c540 (patch)
tree83d7f3bb6d8d70d7e7471917f1434cd2571a9c63 /src/hls/Abstr.v
parenta64b65a9f5b52372b413c31873fa14c3b1785b00 (diff)
downloadvericert-db4da00aea8b51bc9d90d83f981b9163eec3c540.tar.gz
vericert-db4da00aea8b51bc9d90d83f981b9163eec3c540.zip
Work on CondElim proof
Diffstat (limited to 'src/hls/Abstr.v')
-rw-r--r--src/hls/Abstr.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/src/hls/Abstr.v b/src/hls/Abstr.v
index ab0511f..9992b1c 100644
--- a/src/hls/Abstr.v
+++ b/src/hls/Abstr.v
@@ -728,11 +728,11 @@ Definition beq_pred_expr (pe1 pe2: pred_expr) : bool :=
Definition check := Rtree.beq beq_pred_expr.
-Compute (check (empty # (Reg 2) <-
- ((((Pand (Plit (true, 4)) (¬ (Plit (true, 4))))), (Ebase (Reg 9))) ::|
- (NE.singleton (((Plit (true, 2))), (Ebase (Reg 3))))))
- (empty # (Reg 2) <- (NE.singleton (((Por (Plit (true, 2)) (Pand (Plit (true, 3)) (¬ (Plit (true, 3)))))),
- (Ebase (Reg 3)))))).
+(* Compute (check (empty # (Reg 2) <- *)
+(* ((((Pand (Plit (true, 4)) (¬ (Plit (true, 4))))), (Ebase (Reg 9))) ::| *)
+(* (NE.singleton (((Plit (true, 2))), (Ebase (Reg 3)))))) *)
+(* (empty # (Reg 2) <- (NE.singleton (((Por (Plit (true, 2)) (Pand (Plit (true, 3)) (¬ (Plit (true, 3)))))), *)
+(* (Ebase (Reg 3)))))). *)
Lemma inj_asgn_eg : forall a b, (a =? b)%nat = (a =? a)%nat -> a = b.
Proof.