Skip to content

Commit a508423

Browse files
authored
Merge pull request #10 from palmskog/fix-license-opam
Unambiguously state MIT license
2 parents 7e9c895 + 4164f94 commit a508423

File tree

3 files changed

+48
-53
lines changed

3 files changed

+48
-53
lines changed

LibHyps/LibHypsNaming.v

Lines changed: 0 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -2,11 +2,6 @@
22
This file is part of LibHyps. It is distributed under the MIT
33
"expat license". You should have recieved a LICENSE file with it. *)
44

5-
(**************************************************************************
6-
* A user-customizable auto-naming scheme for hypothesis in Coq *
7-
* Author: Pierre Courtieu *
8-
* Distributed under the terms of the LGPL-v3 license *
9-
***************************************************************************)
105
Require Import Arith ZArith List LibHyps.TacNewHyps.
116
Import ListNotations.
127
Local Open Scope list.

coq-libhyps.opam

Lines changed: 48 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,48 @@
1+
# this is a mirror of an opam description file in the
2+
# opam-coq-archive at:
3+
# https://github.com/coq/opam-coq-archive/tree/master/released/packages/coq-libhyps
4+
# the latter being official and probably more up to date.
5+
6+
opam-version: "2.0"
7+
maintainer: "[email protected]"
8+
synopsis: "Hypotheses manipulation library"
9+
10+
homepage: "https://github.com/Matafou/LibHyps"
11+
dev-repo: "git+https://github.com/Matafou/LibHyps.git"
12+
bug-reports: "https://github.com/Matafou/LibHyps/issues"
13+
doc: "https://github.com/Matafou/LibHyps/blob/master/Demo/demo.v"
14+
license: "MIT"
15+
16+
build: [
17+
["./configure.sh"]
18+
[make "-j%{jobs}%"]
19+
]
20+
21+
install: [make "install"]
22+
23+
depends: [
24+
"coq" {(>= "8.11" & < "8.17~") | (= "dev")}
25+
]
26+
27+
tags: [
28+
"keyword:proof environment manipulation"
29+
"keyword:forward reasoning"
30+
"keyword:hypothesis naming"
31+
"category:Miscellaneous/Coq Tactics Library"
32+
"logpath:LibHyps"
33+
]
34+
35+
authors: [
36+
"Pierre Courtieu"
37+
]
38+
39+
description: "
40+
This library defines a set of tactics to manipulate hypothesis
41+
individually or by group. In particular it allows applying a tactic on
42+
each hypothesis of a goal, or only on *new* hypothesis after some
43+
tactic. Examples of manipulations: automatic renaming, subst, revert,
44+
or any tactic expecting a hypothesis name as argument.
45+
46+
It also provides the especialize tactic to ease forward reasoning by
47+
instantianting one, several or all premisses of a hypothesis.
48+
"

opam

Lines changed: 0 additions & 48 deletions
This file was deleted.

0 commit comments

Comments
 (0)