aboutsummaryrefslogtreecommitdiffhomepage
path: root/stm/lemmas.ml
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-06-25 17:04:35 +0200
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-06-25 17:04:35 +0200
commit753b8f4aaa78fe1cf8ea033d8cf45e88b5da9d13 (patch)
tree66ef0fdf8f9152d0740b1f875d80343bac1ae4af /stm/lemmas.ml
parent0a829ad04841d0973b22b4407b95f518276b66e7 (diff)
all coqide specific files moved into ide/
lib/interface split into: - lib/feedback subscribe-based feedback bus (also used by coqidetop) - ide/interface definition of coqide protocol messages lib/pp structured info/err/warn messages lib/serialize split into: - lib/serialize generic xml serialization (list, pairs, int, loc, ...) used by coqide but potentially useful to other interfaces - ide/xmlprotocol serialization of protocol messages as in ide/interface the only drawback is that coqidetop needs -thread and I had to pass that option to all files in ide/
Diffstat (limited to 'stm/lemmas.ml')
-rw-r--r--stm/lemmas.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/stm/lemmas.ml b/stm/lemmas.ml
index c40000811..5d2babaca 100644
--- a/stm/lemmas.ml
+++ b/stm/lemmas.ml
@@ -323,7 +323,7 @@ let standard_proof_terminator compute_guard hook =
let open Proof_global in function
| Admitted ->
admit hook ();
- Pp.feedback Interface.AddedAxiom
+ Pp.feedback Feedback.AddedAxiom
| Proved (is_opaque,idopt,proof) ->
let proof = get_proof proof compute_guard hook is_opaque in
begin match idopt with
@@ -337,7 +337,7 @@ let universe_proof_terminator compute_guard hook =
let open Proof_global in function
| Admitted ->
admit (hook Evd.empty_evar_universe_context) ();
- Pp.feedback Interface.AddedAxiom
+ Pp.feedback Feedback.AddedAxiom
| Proved (is_opaque,idopt,proof) ->
let proof = get_proof proof compute_guard
(hook proof.Proof_global.universes) is_opaque in