Skip to content

Commit

Permalink
Fix flake + adapt to coq/coq#18529
Browse files Browse the repository at this point in the history
Fixing Coq pin in flake and adding correction to make coq master
branch compile.
  • Loading branch information
rtetley committed Feb 6, 2024
1 parent 87dd6d0 commit bf063d8
Show file tree
Hide file tree
Showing 3 changed files with 14 additions and 6 deletions.
8 changes: 4 additions & 4 deletions flake.lock

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

8 changes: 6 additions & 2 deletions flake.nix
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@

flake-utils.url = "github:numtide/flake-utils";

coq-master = { url = "github:coq/coq/fbaea89860348ca2b2ca485e52df7215bea27746"; }; # Should be kept in sync with PIN_COQ in CI workflow
coq-master = { url = "github:coq/coq/b157d65080076498ad04dd3918c1e508eb9740c0"; }; # Should be kept in sync with PIN_COQ in CI workflow
coq-master.inputs.nixpkgs.follows = "nixpkgs";

};
Expand Down Expand Up @@ -156,9 +156,13 @@

devShells.vscoq-language-server-coq-master =
with import nixpkgs { inherit system; };
let ocamlPackages = ocaml-ng.ocamlPackages_4_14; in
mkShell {
buildInputs =
self.packages.${system}.vscoq-language-server-coq-master.buildInputs;
self.packages.${system}.vscoq-language-server-coq-master.buildInputs
++ (with ocamlPackages; [
ocaml-lsp
]);
};

devShells.default =
Expand Down
4 changes: 4 additions & 0 deletions language-server/dm/parTactic.ml
Original file line number Diff line number Diff line change
Expand Up @@ -60,7 +60,11 @@ let assign_tac ~abstract res : unit Proofview.tactic =
tclUNIT ()
end)

[%%if coq = "8.18" || coq = "8.19"]
let command_focus = Proof.new_focus_kind ()
[%%else]
let command_focus = Proof.new_focus_kind "vscoq_command_focus"
[%%endif]

let worker_solve_one_goal { TacticJob.state; ast; goalno; goal } ~send_back =
let focus_cond = Proof.no_cond command_focus in
Expand Down

0 comments on commit bf063d8

Please sign in to comment.