aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--contrib/xml/xmlcommand.ml2
-rw-r--r--library/decl_kinds.ml1
-rw-r--r--toplevel/command.ml3
3 files changed, 2 insertions, 4 deletions
diff --git a/contrib/xml/xmlcommand.ml b/contrib/xml/xmlcommand.ml
index 2157dab56..ba9e87e0b 100644
--- a/contrib/xml/xmlcommand.ml
+++ b/contrib/xml/xmlcommand.ml
@@ -455,7 +455,6 @@ let kind_of_variable id =
| DK.IsAssumption DK.Logical -> "VARIABLE","Hypothesis"
| DK.IsAssumption DK.Conjectural -> "VARIABLE","Conjecture"
| DK.IsDefinition -> "VARIABLE","LocalDefinition"
- | DK.IsConjecture -> "VARIABLE","Conjecture"
| DK.IsProof DK.LocalStatement -> "VARIABLE","LocalFact"
;;
@@ -466,7 +465,6 @@ let kind_of_constant kn =
| DK.IsAssumption DK.Logical -> "AXIOM","Axiom"
| DK.IsAssumption DK.Conjectural -> "AXIOM","Conjecture"
| DK.IsDefinition -> "DEFINITION","Definition"
- | DK.IsConjecture -> "THEOREM","Conjecture"
| DK.IsProof thm -> "THEOREM",kind_of_theorem thm
;;
diff --git a/library/decl_kinds.ml b/library/decl_kinds.ml
index bec9ab7c6..66b1bb072 100644
--- a/library/decl_kinds.ml
+++ b/library/decl_kinds.ml
@@ -61,7 +61,6 @@ type local_theorem_kind = LocalStatement
type 'a mathematical_kind =
| IsAssumption of type_as_formula_kind
| IsDefinition
- | IsConjecture
| IsProof of 'a
type global_kind = theorem_kind mathematical_kind
diff --git a/toplevel/command.ml b/toplevel/command.ml
index 6dad04c98..f2642fcd1 100644
--- a/toplevel/command.ml
+++ b/toplevel/command.ml
@@ -692,7 +692,8 @@ let admit () =
if k <> IsGlobal (Proof Conjecture) then
error "Only statements declared as conjecture can be admitted";
*)
- let (_,kn) = declare_constant id (ParameterEntry typ, IsConjecture) in
+ let (_,kn) =
+ declare_constant id (ParameterEntry typ, IsAssumption Conjectural) in
hook Global (ConstRef kn);
Pfedit.delete_current_proof ();
assumption_message id