aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLBlockInstr.v
diff options
context:
space:
mode:
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 8d3fde4..5162b38 100644
--- a/src/hls/RTLBlockInstr.v
+++ b/src/hls/RTLBlockInstr.v
@@ -348,9 +348,9 @@ Fixpoint init_regs (vl: list val) (rl: list reg) {struct rl} : regset :=
end.
Record instr_state := mk_instr_state {
- instr_st_regset: regset;
- instr_st_predset: predset;
- instr_st_mem: mem;
+ is_rs: regset;
+ is_ps: predset;
+ is_mem: mem;
}.
Section DEFINITION.