diff options
| author | Emilio Jesus Gallego Arias | 2020-04-03 01:16:22 -0400 |
|---|---|---|
| committer | Emilio Jesus Gallego Arias | 2020-04-15 11:12:59 -0400 |
| commit | 38aa25757957e9e9f879509605f06ada5992ca36 (patch) | |
| tree | cc635dc3916971d0615924367cc314226148d55a | |
| parent | 1dc70876b4a5ad027b3b73aa6ba741e89320d17d (diff) | |
[tmp] Compat API for CI
Rewriter needs a bit of work as it calls a removed function, but no
big deal.
| -rw-r--r-- | tactics/declare.mli | 11 | ||||
| -rw-r--r-- | vernac/pfedit.ml | 9 | ||||
| -rw-r--r-- | vernac/proof_global.ml | 7 | ||||
| -rw-r--r-- | vernac/vernac.mllib | 2 |
4 files changed, 29 insertions, 0 deletions
diff --git a/tactics/declare.mli b/tactics/declare.mli index 25dcc84fc8..1fabf80b2a 100644 --- a/tactics/declare.mli +++ b/tactics/declare.mli @@ -301,3 +301,14 @@ val get_current_goal_context : Proof.t -> Evd.evar_map * Environ.env If there is no pending proof then it returns the current global environment and empty evar_map. *) val get_current_context : Proof.t -> Evd.evar_map * Environ.env + +(** Temporarily re-exported for 3rd party code; don't use *) +val build_constant_by_tactic : + name:Names.Id.t -> + ?opaque:opacity_flag -> + uctx:UState.t -> + sign:Environ.named_context_val -> + poly:bool -> + EConstr.types -> + unit Proofview.tactic -> + Evd.side_effects proof_entry * bool * UState.t diff --git a/vernac/pfedit.ml b/vernac/pfedit.ml new file mode 100644 index 0000000000..d6b9592176 --- /dev/null +++ b/vernac/pfedit.ml @@ -0,0 +1,9 @@ +(* Compat API / *) +let get_current_context = Declare.get_current_context +let solve = Proof.solve +let by = Declare.by +let refine_by_tactic = Proof.refine_by_tactic + +(* We don't want to export this anymore, but we do for now *) +let build_by_tactic = Declare.build_by_tactic +let build_constant_by_tactic = Declare.build_constant_by_tactic diff --git a/vernac/proof_global.ml b/vernac/proof_global.ml new file mode 100644 index 0000000000..b6c07042e2 --- /dev/null +++ b/vernac/proof_global.ml @@ -0,0 +1,7 @@ +(* compatibility module; can be removed once we agree on the API *) + +type t = Declare.Proof.t +let map_proof = Declare.Proof.map_proof +let get_proof = Declare.Proof.get_proof + +type opacity_flag = Declare.opacity_flag = Opaque | Transparent diff --git a/vernac/vernac.mllib b/vernac/vernac.mllib index 5a2bdb43d4..b7728fe699 100644 --- a/vernac/vernac.mllib +++ b/vernac/vernac.mllib @@ -44,3 +44,5 @@ ComArguments Vernacentries Vernacstate Vernacinterp +Proof_global +Pfedit |
