aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--Makefile2
-rw-r--r--library/declare.mli5
-rw-r--r--proofs/pfedit.ml2
3 files changed, 2 insertions, 7 deletions
diff --git a/Makefile b/Makefile
index 7d51977c2..11bf94d4e 100644
--- a/Makefile
+++ b/Makefile
@@ -74,7 +74,7 @@ TACTICS=tactics/dn.cmo tactics/termdn.cmo tactics/btermdn.cmo \
tactics/tacentries.cmo tactics/hiddentac.cmo tactics/elim.cmo
TOPLEVEL=toplevel/himsg.cmo toplevel/errors.cmo toplevel/vernacinterp.cmo \
- toplevel/metasyntax.cmo \
+ toplevel/metasyntax.cmo toplevel/command.cmo \
toplevel/vernacentries.cmo toplevel/vernac.cmo toplevel/mltop.cmo \
toplevel/protectedtoplevel.cmo toplevel/toplevel.cmo
diff --git a/library/declare.mli b/library/declare.mli
index 1a9a0fac2..a8848660d 100644
--- a/library/declare.mli
+++ b/library/declare.mli
@@ -21,23 +21,18 @@ type strength =
| NeverDischarge
type variable_declaration = constr * strength * bool
-
val declare_variable : identifier -> variable_declaration -> unit
type constant_declaration = constant_entry * strength * bool
-
val declare_constant : identifier -> constant_declaration -> unit
val declare_parameter : identifier -> constr -> unit
-
val declare_mind : mutual_inductive_entry -> unit
-
val declare_eliminations : section_path -> unit
-
val declare_syntax_constant : identifier -> constr -> unit
val make_strength : string list -> strength
diff --git a/proofs/pfedit.ml b/proofs/pfedit.ml
index a9a8e0d3b..9fc376855 100644
--- a/proofs/pfedit.ml
+++ b/proofs/pfedit.ml
@@ -260,7 +260,7 @@ let start_proof_with_type na str env concl =
let start_proof na str concl_com =
let sigma = Evd.empty in
let env = Global.env() in
- let concl = fconstruct_type sigma (Environ.context env) concl_com in
+ let concl = type_of_com env concl_com in
start_proof_with_type na str env concl.body
let start_proof_constr na str concl =