aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLPargenproof.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-03-24 11:46:15 +0000
committerYann Herklotz <git@yannherklotz.com>2022-03-24 11:46:15 +0000
commit30baa719fb15c45b13cb869056e51ec7446c0207 (patch)
tree35be4ec314fbcdd27adeba367d3bbf5fc844cdd4 /src/hls/RTLPargenproof.v
parentb9e793eef135bd411c9945f0b1ba99308d9edbd5 (diff)
downloadvericert-30baa719fb15c45b13cb869056e51ec7446c0207.tar.gz
vericert-30baa719fb15c45b13cb869056e51ec7446c0207.zip
Add more documentation
Diffstat (limited to 'src/hls/RTLPargenproof.v')
-rw-r--r--src/hls/RTLPargenproof.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/hls/RTLPargenproof.v b/src/hls/RTLPargenproof.v
index 5188709..6d61572 100644
--- a/src/hls/RTLPargenproof.v
+++ b/src/hls/RTLPargenproof.v
@@ -16,7 +16,7 @@
* along with this program. If not, see <https://www.gnu.org/licenses/>.
*)
-(* [[file:../../lit/scheduler.org::rtlpargenproof-imports][rtlpargenproof-imports]] *)
+(* [[file:../../docs/scheduler.org::rtlpargenproof-imports][rtlpargenproof-imports]] *)
Require Import compcert.backend.Registers.
Require Import compcert.common.AST.
Require Import compcert.common.Errors.
@@ -39,7 +39,7 @@ Require Import vericert.hls.Abstr.
#[local] Open Scope pred_op.
(* rtlpargenproof-imports ends here *)
-(* [[file:../../lit/scheduler.org::rtlpargenproof-main][rtlpargenproof-main]] *)
+(* [[file:../../docs/scheduler.org::rtlpargenproof-main][rtlpargenproof-main]] *)
(*Definition is_regs i := match i with mk_instr_state rs _ => rs end.
Definition is_mem i := match i with mk_instr_state _ m => m end.