aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLBlockInstr.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2021-01-29 19:20:07 +0000
committerYann Herklotz <git@yannherklotz.com>2021-01-29 19:20:07 +0000
commitb708486d60c4c0aa695dca4ee46861c87cebb9e1 (patch)
tree89532b748657ded3bf86da3ae15166c42093ace8 /src/hls/RTLBlockInstr.v
parentcd6bf14e8f5ce68624ba20a33b8278c78cb632fb (diff)
downloadvericert-b708486d60c4c0aa695dca4ee46861c87cebb9e1.tar.gz
vericert-b708486d60c4c0aa695dca4ee46861c87cebb9e1.zip
Fix definitions of proofs some more
Diffstat (limited to 'src/hls/RTLBlockInstr.v')
-rw-r--r--src/hls/RTLBlockInstr.v10
1 files changed, 0 insertions, 10 deletions
diff --git a/src/hls/RTLBlockInstr.v b/src/hls/RTLBlockInstr.v
index 2744527..90edc2e 100644
--- a/src/hls/RTLBlockInstr.v
+++ b/src/hls/RTLBlockInstr.v
@@ -202,16 +202,6 @@ Section RELSEM.
(RBstore chunk addr args src)
(InstrState rs m').
- Inductive step_instr_list: val -> instr_state -> list instr -> instr_state -> Prop :=
- | exec_RBcons:
- forall state i state' state'' instrs sp,
- step_instr sp state i state' ->
- step_instr_list sp state' instrs state'' ->
- step_instr_list sp state (i :: instrs) state''
- | exec_RBnil:
- forall state sp,
- step_instr_list sp state nil state.
-
Inductive step_cf_instr: state -> cf_instr -> trace -> state -> Prop :=
| exec_RBcall:
forall s f sp rs m res fd ros sig args pc pc',