aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GiblePargenproof.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2023-06-21 18:57:33 +0100
committerYann Herklotz <git@yannherklotz.com>2023-06-21 18:57:33 +0100
commit4d262face34cb79d478823fd8db32cf02dc187f8 (patch)
tree820335def3dc6d2fda3b779e8079b0c5fac8620c /src/hls/GiblePargenproof.v
parent323f262727ac3a4b129bdaeaa21083d8daa5184c (diff)
downloadvericert-4d262face34cb79d478823fd8db32cf02dc187f8.tar.gz
vericert-4d262face34cb79d478823fd8db32cf02dc187f8.zip
Add SMTCoq solver as dependency
Diffstat (limited to 'src/hls/GiblePargenproof.v')
-rw-r--r--src/hls/GiblePargenproof.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/hls/GiblePargenproof.v b/src/hls/GiblePargenproof.v
index 5d36ae9..b774b48 100644
--- a/src/hls/GiblePargenproof.v
+++ b/src/hls/GiblePargenproof.v
@@ -127,7 +127,7 @@ Qed.
Definition state_lessdef := GiblePargenproofEquiv.match_states.
Definition match_prog (prog : GibleSeq.program) (tprog : GiblePar.program) :=
- match_program (fun cu f tf => transl_fundef f = Errors.OK tf) eq prog tprog.
+ match_program (fun cu f tf => transl_fundef f = OK tf) eq prog tprog.
(* TODO: Fix the `bb` and add matches for them. *)
Inductive match_stackframes: GibleSeq.stackframe -> GiblePar.stackframe -> Prop :=
@@ -177,7 +177,7 @@ Section CORRECTNESS.
forall (b: Values.block) (f: GibleSeq.fundef),
Genv.find_funct_ptr ge b = Some f ->
exists tf,
- Genv.find_funct_ptr tge b = Some tf /\ transl_fundef f = Errors.OK tf.
+ Genv.find_funct_ptr tge b = Some tf /\ transl_fundef f = OK tf.
Proof using TRANSL.
intros. exploit (Genv.find_funct_ptr_match TRANSL); eauto.
intros (cu & tf & P & Q & R); exists tf; auto.
@@ -187,7 +187,7 @@ Section CORRECTNESS.
forall (v: Values.val) (f: GibleSeq.fundef),
Genv.find_funct ge v = Some f ->
exists tf,
- Genv.find_funct tge v = Some tf /\ transl_fundef f = Errors.OK tf.
+ Genv.find_funct tge v = Some tf /\ transl_fundef f = OK tf.
Proof using TRANSL.
intros. exploit (Genv.find_funct_match TRANSL); eauto.
intros (cu & tf & P & Q & R); exists tf; auto.