aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2019-06-06 17:28:26 +0200
committerEmilio Jesus Gallego Arias2019-06-24 20:55:09 +0200
commitda5bbda84bd22b87a6057175c9d4d2391808e294 (patch)
treec65591866875814ca83d99d28330d59dd4518452 /plugins
parent9d65c49f05f946557df4c67b6e752f978e1e9352 (diff)
[api] [proof] Move `discharge` type to vernac_ast where it is used.
This seems like the right location, a bit more refactoring should be possible.
Diffstat (limited to 'plugins')
-rw-r--r--plugins/funind/g_indfun.mlg2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/funind/g_indfun.mlg b/plugins/funind/g_indfun.mlg
index ef9d91c7fa..e20d010c71 100644
--- a/plugins/funind/g_indfun.mlg
+++ b/plugins/funind/g_indfun.mlg
@@ -182,7 +182,7 @@ let is_proof_termination_interactively_checked recsl =
let classify_as_Fixpoint recsl =
Vernac_classifier.classify_vernac
- (Vernacexpr.(CAst.make @@ VernacExpr([], VernacFixpoint(Decl_kinds.NoDischarge, List.map snd recsl))))
+ (Vernacexpr.(CAst.make @@ VernacExpr([], VernacFixpoint(NoDischarge, List.map snd recsl))))
let classify_funind recsl =
match classify_as_Fixpoint recsl with