Skip to content

Commit

Permalink
cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
gares committed Oct 5, 2023
1 parent a065e6f commit 336ee12
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions HB/instance.elpi
Original file line number Diff line number Diff line change
Expand Up @@ -402,7 +402,7 @@ declare-wrapper-inst TheType ML TheMixins TyWP SectionName CSL :- std.do![

pred is-structure-op-w-wrapper i:term.
is-structure-op-w-wrapper (global (const C)) :- exported-op _ _ C, wrapper-mixin _ (const C) _.
is-structure-op-w-wrapper (app[global (const C)|_]) :- std.spy(exported-op _ _ C), wrapper-mixin _ (const C) _.
is-structure-op-w-wrapper (app[global (const C)|_]) :- exported-op _ _ C, wrapper-mixin _ (const C) _.

pred derive-wrapper-instances i:term, i:mixinname, o:term, o:constant.
derive-wrapper-instances Instance WrapperMixin WrapperSubject C :- std.do! [
Expand Down Expand Up @@ -440,7 +440,7 @@ derive-wrapper-instances Instance WrapperMixin WrapperSubject C :- std.do! [

Name is "wrapped__" ^ {std.any->string {new_int}},

std.spy(log.coq.env.add-const-noimplicits Name NewInstance Ty @transparent! C),
log.coq.env.add-const-noimplicits Name NewInstance Ty @transparent! C,
].

pred wrap-a-mixin i:gref, i:mixinname, i:constant, o:term, o:mixinname, o:constant.
Expand Down
2 changes: 1 addition & 1 deletion tests/monoid_enriched_cat.v
Original file line number Diff line number Diff line change
Expand Up @@ -62,7 +62,7 @@ Succeed HB.structure
(forall A B : Obj, isMon (hom A B)) }.

(* which one is best? *)
Fail HB.structure
Succeed HB.structure
Definition Monoid_enriched_quiver :=
{ Obj of isQuiver Obj &
(forall A B : Obj, isMon (@hom (Quiver.clone Obj _) A B)) }.
Expand Down

0 comments on commit 336ee12

Please sign in to comment.