aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/glob_term.ml
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-12-24 23:49:21 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-12-24 23:49:21 +0000
commitd33ced344ba377f0a4003102d77f880fda108fd7 (patch)
treea8f7642bb599a08ada8b6392d0fa14f823e57e3c /pretyping/glob_term.ml
parent6ebd4c4ad28d46965623e72d8654c36fcc6fe9b0 (diff)
More {raw => glob} changes for consistency
perl -pi -e 's/(\W|_)raw((?:sort|_prop|terms?|_branch|_red_flag|pat tern|_constr_of|_of_pat)(?:\W|_))/\1glob_\2/g;s/glob__/glob_/g;s/(\ W)R((?:Prop|Type|Fix|CoFix|StructRec|WfRec|MeasureRec)\W)/\1G\2/g;s /glob_terms?/glob_constr/g' **/*.ml* git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13756 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/glob_term.ml')
-rw-r--r--pretyping/glob_term.ml16
1 files changed, 8 insertions, 8 deletions
diff --git a/pretyping/glob_term.ml b/pretyping/glob_term.ml
index deba9a257..b973a24f7 100644
--- a/pretyping/glob_term.ml
+++ b/pretyping/glob_term.ml
@@ -30,7 +30,7 @@ let cases_pattern_loc = function
type patvar = identifier
-type rawsort = RProp of Term.contents | RType of Univ.universe option
+type glob_sort = GProp of Term.contents | GType of Univ.universe option
type binding_kind = Lib.binding_kind = Explicit | Implicit
@@ -64,18 +64,18 @@ type glob_constr =
| GIf of loc * glob_constr * (name * glob_constr option) * glob_constr * glob_constr
| GRec of loc * fix_kind * identifier array * glob_decl list array *
glob_constr array * glob_constr array
- | GSort of loc * rawsort
+ | GSort of loc * glob_sort
| GHole of (loc * hole_kind)
| GCast of loc * glob_constr * glob_constr cast_type
| GDynamic of loc * Dyn.t
and glob_decl = name * binding_kind * glob_constr option * glob_constr
-and fix_recursion_order = RStructRec | RWfRec of glob_constr | RMeasureRec of glob_constr * glob_constr option
+and fix_recursion_order = GStructRec | GWfRec of glob_constr | GMeasureRec of glob_constr * glob_constr option
and fix_kind =
- | RFix of ((int option * fix_recursion_order) array * int)
- | RCoFix of int
+ | GFix of ((int option * fix_recursion_order) array * int)
+ | GCoFix of int
and predicate_pattern =
name * (loc * inductive * int * name list) option
@@ -366,7 +366,7 @@ let glob_constr_of_closed_cases_pattern = function
(**********************************************************************)
(* Reduction expressions *)
-type 'a raw_red_flag = {
+type 'a glob_red_flag = {
rBeta : bool;
rIota : bool;
rZeta : bool;
@@ -392,8 +392,8 @@ type ('a,'b,'c) red_expr_gen =
| Red of bool
| Hnf
| Simpl of 'c with_occurrences option
- | Cbv of 'b raw_red_flag
- | Lazy of 'b raw_red_flag
+ | Cbv of 'b glob_red_flag
+ | Lazy of 'b glob_red_flag
| Unfold of 'b with_occurrences list
| Fold of 'a list
| Pattern of 'a with_occurrences list