diff options
| author | Emilio Jesus Gallego Arias | 2020-05-25 16:30:20 +0200 |
|---|---|---|
| committer | Emilio Jesus Gallego Arias | 2020-06-26 14:38:11 +0200 |
| commit | b143d124e140628e5974da4af1b8a70a4d534598 (patch) | |
| tree | 3e105d09b0c6490cb1b9d1fe185e4eab68ef957e /plugins/derive | |
| parent | a6d663c85d71b3cce007af23419e8030b8c5ac88 (diff) | |
[declare] Move udecl to Info structure.
Diffstat (limited to 'plugins/derive')
| -rw-r--r-- | plugins/derive/derive.ml | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/derive/derive.ml b/plugins/derive/derive.ml index c4f7638fb9..7779e4f4c7 100644 --- a/plugins/derive/derive.ml +++ b/plugins/derive/derive.ml @@ -41,6 +41,6 @@ let start_deriving f suchthat name : Declare.Proof.t = in let info = Declare.Info.make ~proof_ending:(Declare.Proof_ending.(End_derive {f; name})) ~kind () in - let lemma = Declare.start_dependent_proof ~name ~poly ~info ~udecl:UState.default_univ_decl goals in + let lemma = Declare.start_dependent_proof ~name ~poly ~info goals in Declare.Proof.map lemma ~f:(fun p -> Util.pi1 @@ Proof.run_tactic env Proofview.(tclFOCUS 1 2 shelve) p) |
