aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLBlockgen.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-03-28 12:13:09 +0100
committerYann Herklotz <git@yannherklotz.com>2022-03-28 12:13:09 +0100
commitaed203ab3eeea43d84f4e50c5720111208ba7881 (patch)
treec62b5af82c82b25c55ef6467744b01652c194e30 /src/hls/RTLBlockgen.v
parent34e0f092551fcd7e1eef4a8a3c863fa940dcbf2f (diff)
downloadvericert-aed203ab3eeea43d84f4e50c5720111208ba7881.tar.gz
vericert-aed203ab3eeea43d84f4e50c5720111208ba7881.zip
Add specification for RTLBlockgenproof
Diffstat (limited to 'src/hls/RTLBlockgen.v')
-rw-r--r--src/hls/RTLBlockgen.v6
1 files changed, 4 insertions, 2 deletions
diff --git a/src/hls/RTLBlockgen.v b/src/hls/RTLBlockgen.v
index a29709b..dc65cc2 100644
--- a/src/hls/RTLBlockgen.v
+++ b/src/hls/RTLBlockgen.v
@@ -19,6 +19,8 @@
===========
RTLBlockgen
===========
+
+.. coq:: none
|*)
Require compcert.backend.RTL.
@@ -34,8 +36,6 @@ Require Import vericert.hls.RTLBlock.
#[local] Open Scope positive.
-Parameter partition : RTL.function -> Errors.res function.
-
(*|
``find_block max nodes index``: Does not need to be sorted, because we use
filter and the max fold function to find the desired element.
@@ -171,6 +171,8 @@ Definition check_present_blocks (c: code) (n: list positive) (max: positive) (i:
| None => false
end.
+Parameter partition : RTL.function -> Errors.res function.
+
Definition transl_function (f: RTL.function) :=
match partition f with
| Errors.OK f' =>