aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp/coqlib.ml
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-28 19:09:32 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-28 19:09:32 +0000
commit133ce76b38344b062699cc418e59d400becf27b4 (patch)
tree8c57adb725ec8d711e18d94f388af5989ca97e41 /interp/coqlib.ml
parent836cf5e7ea5a83845cd70e3ba3a03db3f736e555 (diff)
Notation concise pour la valeur par défaut des cas reconnus comme
impossibles dans un filtrage dépendant. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11014 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'interp/coqlib.ml')
-rw-r--r--interp/coqlib.ml8
1 files changed, 8 insertions, 0 deletions
diff --git a/interp/coqlib.ml b/interp/coqlib.ml
index ca3347dbb..73614797a 100644
--- a/interp/coqlib.ml
+++ b/interp/coqlib.ml
@@ -109,6 +109,14 @@ let arith_module = make_dir ["Coq";"Arith";"Arith"]
(* TODO: temporary hack *)
let make_kn dir id = Libnames.encode_kn dir id
+let make_con dir id = Libnames.encode_con dir id
+
+(** Identity *)
+
+let id = make_con datatypes_module (id_of_string "id")
+let type_of_id = make_con datatypes_module (id_of_string "ID")
+
+let _ = Cases.set_impossible_default_clause (mkConst id,mkConst type_of_id)
(** Natural numbers *)
let nat_kn = make_kn datatypes_module (id_of_string "nat")