aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/GiblePargenproofCommon.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2023-07-11 15:45:59 +0100
committerYann Herklotz <git@yannherklotz.com>2023-07-11 16:25:09 +0100
commit93117b6e766c25c5aeecdc20a963d5114fb91e59 (patch)
tree60e77f4d09548b3fa077d96e7d0e26fd8b0ad1ef /src/hls/GiblePargenproofCommon.v
parent6cdb6490437b9e609afbf5e8749b24d31c02fce1 (diff)
downloadvericert-93117b6e766c25c5aeecdc20a963d5114fb91e59.tar.gz
vericert-93117b6e766c25c5aeecdc20a963d5114fb91e59.zip
Add equivalence classes
Diffstat (limited to 'src/hls/GiblePargenproofCommon.v')
-rw-r--r--src/hls/GiblePargenproofCommon.v25
1 files changed, 0 insertions, 25 deletions
diff --git a/src/hls/GiblePargenproofCommon.v b/src/hls/GiblePargenproofCommon.v
index 345836f..9254a3b 100644
--- a/src/hls/GiblePargenproofCommon.v
+++ b/src/hls/GiblePargenproofCommon.v
@@ -210,31 +210,6 @@ Proof.
econstructor. split. constructor. right. eauto. auto.
Qed.
-Definition predicated_not_inP {A} (p: Gible.predicate) (l: predicated A) :=
- forall op e, NE.In (op, e) l -> ~ PredIn p op.
-
-Lemma predicated_not_inP_cons :
- forall A p (a: (pred_op * A)) l,
- predicated_not_inP p (NE.cons a l) ->
- predicated_not_inP p l.
-Proof.
- unfold predicated_not_inP; intros. eapply H. econstructor. right; eauto.
-Qed.
-
-Lemma predicated_not_inP_equiv :
- forall A (a: predicated A) p,
- predicated_not_in p a = true -> predicated_not_inP p a.
-Proof.
- induction a.
- - intros. cbn in *. unfold predicated_not_inP; intros.
- unfold not; intros. inv H0. cbn in *.
- destruct (predin peq p op) eqn:?; try discriminate. eapply predin_PredIn in H1.
- rewrite H1 in Heqb. discriminate.
- - intros. cbn in H. eapply andb_prop in H. inv H. eapply IHa in H0.
- unfold predicated_not_inP in *; intros. inv H. inv H3; cbn in *; eauto.
- unfold not; intros. eapply predin_PredIn in H. now rewrite H in H1.
-Qed.
-
Lemma truthy_dec:
forall ps a, truthy ps a \/ falsy ps a.
Proof.