Skip to content

Commit

Permalink
[core-dev] coq-stdlib install, take 2
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed Dec 13, 2024
1 parent f5817fd commit e8aa5b2
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion core-dev/packages/coq-stdlib/coq-stdlib.dev/opam
Original file line number Diff line number Diff line change
Expand Up @@ -42,7 +42,9 @@ build: [
"@runtest" {with-test}
"@doc" {with-doc}
]
["dune" "install" name]
]
install: [
["dune" "install" "-p" name "--create-install-files" name]
["sh" "-c" "echo 'From Stdlib Require Import Reals.' > test.v && coqc test.v"] {with-test}
]

Expand Down

0 comments on commit e8aa5b2

Please sign in to comment.