aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GibleSeqgen.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-05-27 01:05:32 +0100
committerYann Herklotz <git@yannherklotz.com>2022-05-27 01:05:32 +0100
commit0a44da6a7037d9eb270386eeef4f929177c4ec0d (patch)
treeac08c768bbdedda7d791972ee0e2c4db1fb5ac14 /src/hls/GibleSeqgen.v
parent27714f85233e52978caebd67b550bde51e693d48 (diff)
downloadvericert-0a44da6a7037d9eb270386eeef4f929177c4ec0d.tar.gz
vericert-0a44da6a7037d9eb270386eeef4f929177c4ec0d.zip
Rewrite a lot fixing scheduling of Gible
Diffstat (limited to 'src/hls/GibleSeqgen.v')
-rw-r--r--src/hls/GibleSeqgen.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/hls/GibleSeqgen.v b/src/hls/GibleSeqgen.v
index 8d52339..31dabf8 100644
--- a/src/hls/GibleSeqgen.v
+++ b/src/hls/GibleSeqgen.v
@@ -42,7 +42,7 @@ Definition check_valid_node (tc: code) (e: node) :=
| _ => false
end.
-Fixpoint check_code (c: RTL.code) (tc: code) (pc: node) (b: BB.t) :=
+Fixpoint check_code (c: RTL.code) (tc: code) (pc: node) (b: SeqBB.t) :=
match c ! pc, b with
| Some (RTL.Inop pc'), RBnop :: (_ :: _ :: _) as b' =>
check_code c tc pc' b'