aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-11 20:03:05 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-11 20:03:05 +0000
commit7f7fa0184ea32c81e77d34683bca8e456b80a19a (patch)
tree6480027178a4e50c5ecc1980f93d52b1d69612b9 /kernel
parent9386577e2f67c49c2c7b6bab00cd6dc4a5b3b513 (diff)
Renommage des find_m*type
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@693 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/inductive.ml4
-rw-r--r--kernel/inductive.mli8
2 files changed, 6 insertions, 6 deletions
diff --git a/kernel/inductive.ml b/kernel/inductive.ml
index 257305b00..1f1312887 100644
--- a/kernel/inductive.ml
+++ b/kernel/inductive.ml
@@ -198,14 +198,14 @@ let find_mrectype env sigma c =
| IsMutInd ind -> (ind, l)
| _ -> raise Induc
-let find_minductype env sigma c =
+let find_inductive env sigma c =
let (t, l) = whd_betadeltaiota_stack env sigma c in
match kind_of_term t with
| IsMutInd ((sp,i),_ as ind)
when mind_type_finite (lookup_mind sp env) i -> (ind, l)
| _ -> raise Induc
-let find_mcoinductype env sigma c =
+let find_coinductive env sigma c =
let (t, l) = whd_betadeltaiota_stack env sigma c in
match kind_of_term t with
| IsMutInd ((sp,i),_ as ind)
diff --git a/kernel/inductive.mli b/kernel/inductive.mli
index 4f27c30b8..45542ddc3 100644
--- a/kernel/inductive.mli
+++ b/kernel/inductive.mli
@@ -139,14 +139,14 @@ exception Induc
val extract_mrectype : constr -> inductive * constr list
(* [find_m*type env sigma c] coerce [c] to an recursive type (I args).
- [find_mrectype], [find_minductype] and [find_mcoinductype]
+ [find_rectype], [find_inductive] and [find_coinductive]
respectively accepts any recursive type, only an inductive type and
only a coinductive type.
They raise [Induc] if not convertible to a recursive type. *)
-val find_mrectype : env -> 'a evar_map -> constr -> inductive * constr list
-val find_minductype : env -> 'a evar_map -> constr -> inductive * constr list
-val find_mcoinductype : env -> 'a evar_map -> constr -> inductive * constr list
+val find_mrectype : env -> 'a evar_map -> constr -> inductive * constr list
+val find_inductive : env -> 'a evar_map -> constr -> inductive * constr list
+val find_coinductive : env -> 'a evar_map -> constr -> inductive * constr list
val lookup_mind_specif : inductive -> env -> inductive_instance