aboutsummaryrefslogtreecommitdiffstats
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2021-09-19 14:03:18 +0100
committerYann Herklotz <git@yannherklotz.com>2021-09-19 14:03:18 +0100
commit660f82f83c18c672d486baa3429e19a7b77ab4fb (patch)
treee122c92bfbbab5a8df54b74e7eae9d1ea247680e
parent36f5e941da855652310e09a72fbba5a433865f05 (diff)
downloadvericert-dev-michalis.tar.gz
vericert-dev-michalis.zip
Fix infinite loop in proofdev-michalis
-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 20dbbbf..5bfa1f0 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.
@@ -2088,7 +2088,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.