aboutsummaryrefslogtreecommitdiff
path: root/plugins/ltac
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-05-25 16:43:01 +0200
committerEmilio Jesus Gallego Arias2020-06-26 14:38:11 +0200
commit030bb57d4b7e70d45379cab61903b75bf7a41b19 (patch)
treed69b91d1210cb129626a8deeaca6a2d1bf6fad39 /plugins/ltac
parentb143d124e140628e5974da4af1b8a70a4d534598 (diff)
[declare] Reify Proof.t API into the Proof module.
This is in preparation for the next commit which will clean-up the current API flow in `Declare`.
Diffstat (limited to 'plugins/ltac')
-rw-r--r--plugins/ltac/rewrite.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/plugins/ltac/rewrite.ml b/plugins/ltac/rewrite.ml
index 0c1c763b64..405fe7b844 100644
--- a/plugins/ltac/rewrite.ml
+++ b/plugins/ltac/rewrite.ml
@@ -2000,8 +2000,8 @@ let add_morphism_interactive atts m n : Declare.Proof.t =
let info = Declare.Info.make ~hook ~kind () in
Flags.silently
(fun () ->
- let lemma = Declare.start_proof ~name:instance_id ~poly ~info ~impargs:[] evd morph in
- fst (Declare.by (Tacinterp.interp tac) lemma)) ()
+ let lemma = Declare.Proof.start ~name:instance_id ~poly ~info ~impargs:[] evd morph in
+ fst (Declare.Proof.by (Tacinterp.interp tac) lemma)) ()
let add_morphism atts binders m s n =
init_setoid ();