aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/Gible.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2023-04-27 11:44:58 +0100
committerYann Herklotz <git@yannherklotz.com>2023-04-27 11:45:05 +0100
commit405e822a4e769969ef01a683d486accee0d71da2 (patch)
tree986d3e660f621e9d17c621e3c5d3924de1c942cb /src/hls/Gible.v
parenta04e972f3dcc94459399e4d4168b8d26d32e1fae (diff)
downloadvericert-405e822a4e769969ef01a683d486accee0d71da2.tar.gz
vericert-405e822a4e769969ef01a683d486accee0d71da2.zip
Change nat to positive in Sat proof
Diffstat (limited to 'src/hls/Gible.v')
-rw-r--r--src/hls/Gible.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/src/hls/Gible.v b/src/hls/Gible.v
index cc35640..d04c78a 100644
--- a/src/hls/Gible.v
+++ b/src/hls/Gible.v
@@ -156,16 +156,16 @@ Definition regset := Regmap.t val.
Definition predset := PMap.t bool.
Definition eval_predf (pr: predset) (p: pred_op) :=
- sat_predicate p (fun x => pr !! (Pos.of_nat x)).
+ sat_predicate p (fun x => pr !! x).
Lemma sat_pred_agree0 :
forall a b p,
- (forall x, x <> 0%nat -> a x = b x) ->
+ (forall x, a x = b x) ->
sat_predicate p a = sat_predicate p b.
Proof.
induction p; auto; intros.
- - destruct p. cbn. assert (Pos.to_nat p <> 0%nat) by lia.
- apply H in H0. now rewrite H0.
+ - destruct p. cbn.
+ now rewrite H.
- specialize (IHp1 H). specialize (IHp2 H).
cbn. rewrite IHp1. rewrite IHp2. auto.
- specialize (IHp1 H). specialize (IHp2 H).
@@ -210,7 +210,7 @@ Lemma eval_predf_not_PredIn :
eval_predf (ps # p <- b) op = eval_predf ps op.
Proof.
induction op; auto.
- - intros. destruct p0. cbn. rewrite Pos2Nat.id.
+ - intros. destruct p0. cbn.
destruct (peq p p0); subst.
{ exfalso; apply H; constructor. }
rewrite Regmap.gso; auto.