Skip to content

Commit

Permalink
Compat typeclass for list_reifyl
Browse files Browse the repository at this point in the history
  • Loading branch information
SkySkimmer committed Nov 21, 2023
1 parent ea815c1 commit 3b1b653
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions theories/setoid_ring/Ncring_tac.v
Original file line number Diff line number Diff line change
Expand Up @@ -130,6 +130,11 @@ Ltac list_reifyl0 lterm :=
list_reifyl lvar lterm
end.

Class ReifyL {R:Type} (lvar lterm : list R) := list_reifyl : (list R * list (PExpr Z)).
Arguments list_reifyl {R lvar lterm _}.

Global Hint Extern 0 (ReifyL ?lvar ?lterm) => let reif := list_reifyl lvar lterm in exact reif : typeclass_instances.

Unset Implicit Arguments.

Ltac lterm_goal g :=
Expand Down

0 comments on commit 3b1b653

Please sign in to comment.