aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/extraction/table.ml
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-10-06 15:48:15 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-10-06 15:48:15 +0000
commitb36e75cca2ea910dead09864c4f10ba79b894a35 (patch)
treebd2830f5635f091f04168acda4623d6c9a9afbea /plugins/extraction/table.ml
parent317700df92b77552dfe5709134e1a024cea97812 (diff)
Extraction: allow to use Extraction Inline / NoInline even from under a section.
in addition, a makefile entry pluginsopt for compiling only the .cmxs git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13509 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/extraction/table.ml')
-rw-r--r--plugins/extraction/table.ml3
1 files changed, 2 insertions, 1 deletions
diff --git a/plugins/extraction/table.ml b/plugins/extraction/table.ml
index c1b488f35..c22bb17ea 100644
--- a/plugins/extraction/table.ml
+++ b/plugins/extraction/table.ml
@@ -482,6 +482,8 @@ let inline_extraction =
cache_function = (fun (_,(b,l)) -> add_inline_entries b l);
load_function = (fun _ (_,(b,l)) -> add_inline_entries b l);
classify_function = (fun o -> Substitute o);
+ discharge_function =
+ (fun (_,(b,l)) -> Some (b, List.map pop_global_reference l));
subst_function =
(fun (s,(b,l)) -> (b,(List.map (fun x -> fst (subst_global s x)) l)))
}
@@ -494,7 +496,6 @@ let _ = declare_summary "Extraction Inline"
(* Grammar entries. *)
let extraction_inline b l =
- check_inside_section ();
let refs = List.map Nametab.global l in
List.iter
(fun r -> match r with