aboutsummaryrefslogtreecommitdiffhomepage
path: root/vernac/comAssumption.ml
diff options
context:
space:
mode:
authorGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2018-04-02 04:26:09 +0200
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2018-04-06 02:59:34 +0200
commit79ff2bc044aa86a5ce30f0c24647db8c8e2544fa (patch)
treeab262754c02841288ce18020bb03b28974f4858a /vernac/comAssumption.ml
parentb7938d0a51cdef8076bf5e1a58907b845a3fcc3d (diff)
[api] Remove dependency of library on Vernacexpr.
Morally, `library` should not depend on the vernacular definition. This will also create problems when trying to modularize the codebase due to the cycle [vernacs depend for example on constrexprs]. The fix is fortunately easy.
Diffstat (limited to 'vernac/comAssumption.ml')
-rw-r--r--vernac/comAssumption.ml3
1 files changed, 1 insertions, 2 deletions
diff --git a/vernac/comAssumption.ml b/vernac/comAssumption.ml
index 6a590758f..26a46a752 100644
--- a/vernac/comAssumption.ml
+++ b/vernac/comAssumption.ml
@@ -20,7 +20,6 @@ open Constrintern
open Impargs
open Decl_kinds
open Pretyping
-open Vernacexpr
open Entries
(* 2| Variable/Hypothesis/Parameter/Axiom declarations *)
@@ -66,7 +65,7 @@ match local with
| Global | Local | Discharge ->
let do_instance = should_axiom_into_instance local in
let local = DeclareDef.get_locality ident ~kind:"axiom" local in
- let inl = match nl with
+ let inl = let open Declaremods in match nl with
| NoInline -> None
| DefaultInline -> Some (Flags.get_inline_level())
| InlineAt i -> Some i