aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/HTL.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2021-02-15 00:06:29 +0000
committerYann Herklotz <git@yannherklotz.com>2021-02-15 00:06:29 +0000
commit171b326ade18ab77eb155a9d203f2f523708b29b (patch)
treedf9f02bc68c7dc539a67ac376ad7a5d4435c07c3 /src/hls/HTL.v
parent5f1e7aa8fbc4a0e04d0b137410c13f3d8da4d987 (diff)
downloadvericert-171b326ade18ab77eb155a9d203f2f523708b29b.tar.gz
vericert-171b326ade18ab77eb155a9d203f2f523708b29b.zip
Add beginning to scheduling division
Diffstat (limited to 'src/hls/HTL.v')
-rw-r--r--src/hls/HTL.v12
1 files changed, 8 insertions, 4 deletions
diff --git a/src/hls/HTL.v b/src/hls/HTL.v
index c8a0041..d91a340 100644
--- a/src/hls/HTL.v
+++ b/src/hls/HTL.v
@@ -27,16 +27,19 @@ Require compcert.lib.Integers.
Require Import compcert.lib.Maps.
Require Import vericert.common.Vericertlib.
-Require Import vericert.hls.ValueInt.
-Require Import vericert.hls.AssocMap.
Require Import vericert.hls.Array.
+Require Import vericert.hls.AssocMap.
+Require Import vericert.hls.FunctionalUnits.
+Require Import vericert.hls.ValueInt.
Require vericert.hls.Verilog.
-(** The purpose of the hardware transfer language (HTL) is to create a more
+(*|
+The purpose of the hardware transfer language (HTL) is to create a more
hardware-like layout that is still similar to the register transfer language
(RTL) that it came from. The main change is that function calls become module
instantiations and that we now describe a state machine instead of a
-control-flow graph. *)
+control-flow graph.
+|*)
Local Open Scope assocmap.
@@ -65,6 +68,7 @@ Record module: Type :=
mod_start : reg;
mod_reset : reg;
mod_clk : reg;
+ mod_funct_units: funct_units;
mod_scldecls : AssocMap.t (option Verilog.io * Verilog.scl_decl);
mod_arrdecls : AssocMap.t (option Verilog.io * Verilog.arr_decl);
mod_wf : (map_well_formed mod_controllogic /\ map_well_formed mod_datapath);