aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/RTLPargenproof.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2022-03-23 09:47:56 +0000
committerYann Herklotz <git@yannherklotz.com>2022-03-23 09:47:56 +0000
commitf00a195ac17fe47047fafc183663a96ec4125f0d (patch)
treef0c535c0e0b911abb8cf8f6738ee9a05d9d09971 /src/hls/RTLPargenproof.v
parent6b2e01e97ca67219465b92e0fbe536bf2a5434e7 (diff)
downloadvericert-f00a195ac17fe47047fafc183663a96ec4125f0d.tar.gz
vericert-f00a195ac17fe47047fafc183663a96ec4125f0d.zip
Change origin of tangled files
Diffstat (limited to 'src/hls/RTLPargenproof.v')
-rw-r--r--src/hls/RTLPargenproof.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/hls/RTLPargenproof.v b/src/hls/RTLPargenproof.v
index 7b262db..5188709 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/scheduling.org::rtlpargenproof-imports][rtlpargenproof-imports]] *)
+(* [[file:../../lit/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/scheduling.org::rtlpargenproof-main][rtlpargenproof-main]] *)
+(* [[file:../../lit/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.
@@ -1092,7 +1092,7 @@ Proof. induction 2; try rewrite H; eauto with barg. Qed.
eauto. eauto. simplify. eauto. eauto. }
{ unfold bind in *. inv TRANSL0. clear Learn. inv H0. destruct_match; crush.
inv H2. unfold transl_function in Heqr. destruct_match; crush.
- inv Heqr.
+ inv Heqr.
repeat econstructor; eauto.
unfold bind in *. destruct_match; crush. }
{ inv TRANSL0. repeat econstructor; eauto using Events.external_call_symbols_preserved, symbols_preserved, senv_preserved, Events.E0_right. }