aboutsummaryrefslogtreecommitdiffstats
path: root/src/spl/Assumptions.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/spl/Assumptions.v')
-rw-r--r--src/spl/Assumptions.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/src/spl/Assumptions.v b/src/spl/Assumptions.v
index 0a8d79e..102148d 100644
--- a/src/spl/Assumptions.v
+++ b/src/spl/Assumptions.v
@@ -65,7 +65,7 @@ Section Checker.
End Forallb2.
Definition check_hole (s:S.t) (prem_id:list clause_id) (prem:list C.t) (concl:C.t) : C.t :=
- if forallb2 (fun id c => forallb2 (fun i j => i == j) (S.get s id) (S.sort_uniq c)) prem_id prem
+ if forallb2 (fun id c => forallb2 (fun i j => i =? j) (S.get s id) (S.sort_uniq c)) prem_id prem
then concl
else C._true.
@@ -89,7 +89,7 @@ Section Checker_correct.
t_form).
Lemma interp_check_clause c1 : forall c2,
- forallb2 (fun i j => i == j) c1 c2 -> C.interp rho c1 = C.interp rho c2.
+ forallb2 (fun i j => i =? j) c1 c2 -> C.interp rho c1 = C.interp rho c2.
Proof.
induction c1 as [ |l1 c1 IHc1]; simpl; intros [ |l2 c2]; simpl; auto; try discriminate.
unfold is_true. rewrite andb_true_iff. intros [H1 H2].
@@ -97,7 +97,7 @@ Section Checker_correct.
Qed.
Lemma valid_check_clause cid c :
- forallb2 (fun i j => i == j) (S.get s cid) (S.sort_uniq c) ->
+ forallb2 (fun i j => i =? j) (S.get s cid) (S.sort_uniq c) ->
interp_uf rho c.
Proof.
intro H. rewrite <- interp_equiv, <- S.sort_uniq_correct; auto.
@@ -131,7 +131,7 @@ Section Checker_correct.
- unfold C.valid. now rewrite interp_equiv.
- now apply C.interp_true.
- now apply C.interp_true.
- - case_eq (forallb2 (fun i j => i == j) (S.get s pid) (S.sort_uniq p));
+ - case_eq (forallb2 (fun i j => i =? j) (S.get s pid) (S.sort_uniq p));
simpl; intro Heq; [ |now apply C.interp_true].
apply IHpids. apply H. apply (valid_check_clause _ _ Heq).
Qed.