aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/HTLgenproof.v
diff options
context:
space:
mode:
authorMichalis Pardalos <m.pardalos@gmail.com>2021-09-19 18:05:04 +0100
committerMichalis Pardalos <m.pardalos@gmail.com>2021-09-19 18:05:04 +0100
commita56c0bd55f921f85ddbb8b02c2f4c7ac89bf3aaf (patch)
treee0a727e7286bd8199315764aaf9713c35513f606 /src/hls/HTLgenproof.v
parent963aff77e8cb73116bdc4b0250dbd61c787159d2 (diff)
parent660f82f83c18c672d486baa3429e19a7b77ab4fb (diff)
downloadvericert-a56c0bd55f921f85ddbb8b02c2f4c7ac89bf3aaf.tar.gz
vericert-a56c0bd55f921f85ddbb8b02c2f4c7ac89bf3aaf.zip
Merge remote-tracking branch 'upstream/dev-michalis' into dev-michalis
Diffstat (limited to 'src/hls/HTLgenproof.v')
-rw-r--r--src/hls/HTLgenproof.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/hls/HTLgenproof.v b/src/hls/HTLgenproof.v
index 2403f40..13a4345 100644
--- a/src/hls/HTLgenproof.v
+++ b/src/hls/HTLgenproof.v
@@ -646,8 +646,8 @@ Section CORRECTNESS.
forall (s: AST.ident), Genv.find_symbol tge s = Genv.find_symbol ge s.
Proof. intros. eapply (Genv.find_symbol_match TRANSL'). Qed.
- Lemma function_ptr_translated:
- forall (b: Values.block) (f: RTL.fundef),
+ Lemma function_ptr_translated :
+ forall (b : Values.block) (f: RTL.fundef),
Genv.find_funct_ptr ge b = Some f ->
exists tf,
Genv.find_funct_ptr tge b = Some tf /\ transl_fundef prog f = Errors.OK tf.
@@ -2115,7 +2115,7 @@ Section CORRECTNESS.
| [ _ : context[if ?x then _ else _] |- _ ] =>
let EQ := fresh "EQ" in
destruct x eqn:EQ; simpl in *
- | [ H : ret _ _ = _ |- _ ] => invert H
+ | [ H : ret _ = _ |- _ ] => invert H
| [ _ : context[match ?x with | _ => _ end] |- _ ] => destruct x
end.