Skip to content

Commit

Permalink
Fix duplicate names and disable debug auto
Browse files Browse the repository at this point in the history
  • Loading branch information
jaccokrijnen committed Jun 27, 2023
1 parent f0cb01f commit 72e619f
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion src/Language/PlutusIR/Analysis/Equality.v
Original file line number Diff line number Diff line change
Expand Up @@ -170,7 +170,7 @@ Definition string_eqb_eq := String.eqb_eq.
Bool.eqb_true_iff
: reflection.
Definition andb_and : forall s t, s && t = true -> s = true /\ t = true.
Proof. debug auto with reflection. Qed.
Proof. auto with reflection. Qed.

Ltac rewrite_eqbs := repeat (
match goal with
Expand Down
4 changes: 2 additions & 2 deletions src/Language/PlutusIR/Transform/DeadCode.v
Original file line number Diff line number Diff line change
Expand Up @@ -53,7 +53,7 @@ Inductive elim : Term -> Term -> Prop :=


with elim_bindings : list Binding -> list Binding -> Prop :=
| elim_bindings : forall bs bs' bsn bs'n,
| elim_bindings_pure : forall bs bs' bsn bs'n,
bsn = map name_Binding bs ->
bs'n = map name_Binding bs' ->

Expand All @@ -77,7 +77,7 @@ with elim_binding : Binding -> Binding -> Prop :=
elim t t' ->
elim_binding (TermBind s vd t) (TermBind s vd t')

| elim_binding : forall b,
| elim_binding_refl : forall b,
elim_binding b b
.

Expand Down
2 changes: 1 addition & 1 deletion src/Language/PlutusIR/Transform/DeadCode/DecideSound.v
Original file line number Diff line number Diff line change
Expand Up @@ -123,7 +123,7 @@ Proof with eauto with Hints_bindings.
simpl in H.
unfold dec_elim_Bindings in H.
split_hypos.
eapply elim_bindings...
eapply elim_bindings_pure...
Qed.


Expand Down

0 comments on commit 72e619f

Please sign in to comment.