aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLBlockInstr.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2021-07-11 15:59:21 +0200
committerYann Herklotz <git@yannherklotz.com>2021-07-11 15:59:21 +0200
commit178a7c4781c96857fe0a33c777da83e769516152 (patch)
treecf4b5248a144289c84161a6fd73de37523c9d373 /src/hls/RTLBlockInstr.v
parent3dfc30619a4f3ecf0f262481a0891259c2b37ed1 (diff)
downloadvericert-178a7c4781c96857fe0a33c777da83e769516152.tar.gz
vericert-178a7c4781c96857fe0a33c777da83e769516152.zip
Remove unnecessary files and proofs
Diffstat (limited to 'src/hls/RTLBlockInstr.v')
-rw-r--r--src/hls/RTLBlockInstr.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/hls/RTLBlockInstr.v b/src/hls/RTLBlockInstr.v
index 86f8eba..5e123a3 100644
--- a/src/hls/RTLBlockInstr.v
+++ b/src/hls/RTLBlockInstr.v
@@ -211,9 +211,9 @@ Fixpoint trans_pred (bound: nat) (p: pred_op) :
- apply orb_true_intro.
apply satFormula_mult2 in H. inv H. apply i in H0. auto.
apply i0 in H0. auto.
-Admitted.
+Abort.
-Definition sat_pred (bound: nat) (p: pred_op) :
+(*Definition sat_pred (bound: nat) (p: pred_op) :
option ({al : alist | sat_predicate p (interp_alist al) = true}
+ {forall a : asgn, sat_predicate p a = false}).
refine
@@ -243,7 +243,7 @@ Definition sat_pred_temp (bound: nat) (p: pred_op) :=
match trans_pred_temp bound p with
| Some fm => boundedSatSimple bound fm
| None => None
- end.
+ end.*)
Inductive instr : Type :=
| RBnop : instr