Skip to content

Commit

Permalink
Remove tactic param in favor of trocq
Browse files Browse the repository at this point in the history
  • Loading branch information
CohenCyril committed Jan 2, 2024
1 parent 38792d2 commit aafb249
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 4 deletions.
2 changes: 1 addition & 1 deletion examples/Example.v
Original file line number Diff line number Diff line change
Expand Up @@ -51,5 +51,5 @@ Goal
(* forall (X : forall (A : Type@{i}), A -> Type@{i}) (A : Type@{i}) (a : A), A -> X A a -> A. *)
(* forall (T : (Type@{i} -> Type@{j})) (F : ((Type@{i} -> Type@{j}) -> Type@{k})), F T. *)
Proof.
param.
trocq.
Abort.
5 changes: 2 additions & 3 deletions theories/Param.v
Original file line number Diff line number Diff line change
Expand Up @@ -140,7 +140,7 @@ Elpi Query lp:{{
).
}}.

Elpi Tactic param.
Elpi Tactic trocq.
Elpi Accumulate Db trocq.db.
Elpi Accumulate File annot.
Elpi Accumulate File util.
Expand Down Expand Up @@ -201,5 +201,4 @@ Elpi Accumulate lp:{{
}}.
Elpi Typecheck.

Tactic Notation "param" := elpi param.
Tactic Notation "trocq" := elpi param.
Tactic Notation "trocq" := elpi trocq.

0 comments on commit aafb249

Please sign in to comment.