aboutsummaryrefslogtreecommitdiff
path: root/tactics
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2019-07-31 12:04:36 +0200
committerPierre-Marie Pédrot2019-07-31 14:35:23 +0200
commit162eefb562aca2c3741ec24d201deb881663e05a (patch)
treea2da7727bcc10708ce35908cbf75508899bdd862 /tactics
parent94dfb7a578e81641a8b816c9a073b81a1c2e4e88 (diff)
Remove the universe part from the section variable mechanism.
It was factorized away with the universe declaration entry. Actually, pomlymorphic universes were declared twice in Declare, once as a context extension, once as part of the variable itself.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/declare.ml8
1 files changed, 4 insertions, 4 deletions
diff --git a/tactics/declare.ml b/tactics/declare.ml
index b8ba62a5e5..63e9279edc 100644
--- a/tactics/declare.ml
+++ b/tactics/declare.ml
@@ -308,12 +308,12 @@ let declare_variable ~name ~kind d =
if Decls.variable_exists name then
raise (AlreadyDeclared (None, name));
- let impl,opaque,poly,univs = match d with (* Fails if not well-typed *)
+ let impl,opaque,poly = match d with (* Fails if not well-typed *)
| SectionLocalAssum {typ;univs;poly;impl} ->
let () = declare_universe_context ~poly univs in
let () = Global.push_named_assum (name,typ) in
let impl = if impl then Decl_kinds.Implicit else Decl_kinds.Explicit in
- impl, true, poly, univs
+ impl, true, poly
| SectionLocalDef (de) ->
(* The body should already have been forced upstream because it is a
section-local definition, but it's not enforced by typing *)
@@ -338,10 +338,10 @@ let declare_variable ~name ~kind d =
} in
let () = Global.push_named_def (name, se) in
Decl_kinds.Explicit, de.proof_entry_opaque,
- poly, univs
+ poly
in
Nametab.push (Nametab.Until 1) (Libnames.make_path DirPath.empty name) (GlobRef.VarRef name);
- add_section_variable ~name ~kind:impl ~poly univs;
+ add_section_variable ~name ~kind:impl ~poly;
Decls.(add_variable_data name {opaque;kind});
add_anonymous_leaf (inVariable ());
Impargs.declare_var_implicits name;