aboutsummaryrefslogtreecommitdiff
path: root/plugins/ltac
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-05-25 16:30:20 +0200
committerEmilio Jesus Gallego Arias2020-06-26 14:38:11 +0200
commitb143d124e140628e5974da4af1b8a70a4d534598 (patch)
tree3e105d09b0c6490cb1b9d1fe185e4eab68ef957e /plugins/ltac
parenta6d663c85d71b3cce007af23419e8030b8c5ac88 (diff)
[declare] Move udecl to Info structure.
Diffstat (limited to 'plugins/ltac')
-rw-r--r--plugins/ltac/rewrite.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/ltac/rewrite.ml b/plugins/ltac/rewrite.ml
index 0bf97fefa6..0c1c763b64 100644
--- a/plugins/ltac/rewrite.ml
+++ b/plugins/ltac/rewrite.ml
@@ -2000,7 +2000,7 @@ 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:[] ~udecl:UState.default_univ_decl evd morph in
+ let lemma = Declare.start_proof ~name:instance_id ~poly ~info ~impargs:[] evd morph in
fst (Declare.by (Tacinterp.interp tac) lemma)) ()
let add_morphism atts binders m s n =