aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLPargenproof.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-02-25 18:32:35 +0000
committerYann Herklotz <git@yannherklotz.com>2022-02-25 18:32:35 +0000
commit5f34267c4bccb471c71fd5698ec49adc99940850 (patch)
treed8d807f9f81bf8bcca9048201e9f7663e4a8c813 /src/hls/RTLPargenproof.v
parent8d71333042d9ed87a80cffd4005daa0a0acc1810 (diff)
downloadvericert-5f34267c4bccb471c71fd5698ec49adc99940850.tar.gz
vericert-5f34267c4bccb471c71fd5698ec49adc99940850.zip
Fix up some more documentation
Diffstat (limited to 'src/hls/RTLPargenproof.v')
-rw-r--r--src/hls/RTLPargenproof.v7
1 files changed, 2 insertions, 5 deletions
diff --git a/src/hls/RTLPargenproof.v b/src/hls/RTLPargenproof.v
index 588f67f..0023edc 100644
--- a/src/hls/RTLPargenproof.v
+++ b/src/hls/RTLPargenproof.v
@@ -46,12 +46,9 @@ Inductive state_lessdef : instr_state -> instr_state -> Prop :=
(forall x, rs1 !! x = rs2 !! x) ->
state_lessdef (mk_instr_state rs1 m1) (mk_instr_state rs2 m1).
-(*|
-RTLBlock to abstract translation
---------------------------------
+(** *** RTLBlock to abstract translation
-Correctness of translation from RTLBlock to the abstract interpretation language.
-|*)
+Correctness of translation from RTLBlock to the abstract interpretation language. *)
Ltac inv_simp :=
repeat match goal with