aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernacexpr.ml
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel/vernacexpr.ml')
-rw-r--r--toplevel/vernacexpr.ml22
1 files changed, 1 insertions, 21 deletions
diff --git a/toplevel/vernacexpr.ml b/toplevel/vernacexpr.ml
index d7091bfa2..122c0b0b2 100644
--- a/toplevel/vernacexpr.ml
+++ b/toplevel/vernacexpr.ml
@@ -15,6 +15,7 @@ open Tacexpr
open Extend
open Genarg
open Symbols
+open Decl_kinds
(* Toplevel control exceptions *)
exception ProtectedLoop
@@ -85,27 +86,6 @@ type showable =
| ExplainProof of int list
| ExplainTree of int list
-type theorem_kind =
- | Theorem
- | Lemma
- | Decl
- | Fact
- | Remark
-
-type definition_kind =
- | Definition
- | LocalDefinition
-
-type goal_kind =
- | StartTheoremProof of theorem_kind
- | StartDefinitionBody of definition_kind
-
-type assumption_kind =
- | AssumptionHypothesis
- | AssumptionVariable
- | AssumptionAxiom
- | AssumptionParameter
-
type comment =
| CommentConstr of constr_ast
| CommentString of string