aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/funind/glob_termops.mli
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-12-25 13:25:59 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-12-25 13:25:59 +0000
commit2c6c48388fa5ce84d66eb92fd9574951628a2c34 (patch)
tree099c838843543d3b457417b10eb4f8b1e9d5657d /plugins/funind/glob_termops.mli
parent240471f4c9dec6b6b1f97901544d04f53c0902c3 (diff)
Rename mkR* smart constructors (mostly in funind)
perl -pi -e 's/(mk)R(Ref|Var|Evar|PatVar|App|Lambda|Prod|LetIn|Case s|LetTuple|If|Rec|Sort|Hole|Cast|Dynamic|Prop|Type|Fix|CoFix|Struct Rec|WfRec|MeasureRec)/\1G\2/g' **/*.ml* git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13758 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/funind/glob_termops.mli')
-rw-r--r--plugins/funind/glob_termops.mli20
1 files changed, 10 insertions, 10 deletions
diff --git a/plugins/funind/glob_termops.mli b/plugins/funind/glob_termops.mli
index 3afb86298..bfd153579 100644
--- a/plugins/funind/glob_termops.mli
+++ b/plugins/funind/glob_termops.mli
@@ -16,16 +16,16 @@ val pattern_to_term : cases_pattern -> glob_constr
Some basic functions to rebuild glob_constr
In each of them the location is Util.dummy_loc
*)
-val mkRRef : Libnames.global_reference -> glob_constr
-val mkRVar : Names.identifier -> glob_constr
-val mkRApp : glob_constr*(glob_constr list) -> glob_constr
-val mkRLambda : Names.name * glob_constr * glob_constr -> glob_constr
-val mkRProd : Names.name * glob_constr * glob_constr -> glob_constr
-val mkRLetIn : Names.name * glob_constr * glob_constr -> glob_constr
-val mkRCases : glob_constr option * tomatch_tuples * cases_clauses -> glob_constr
-val mkRSort : glob_sort -> glob_constr
-val mkRHole : unit -> glob_constr (* we only build Evd.BinderType Anonymous holes *)
-val mkRCast : glob_constr* glob_constr -> glob_constr
+val mkGRef : Libnames.global_reference -> glob_constr
+val mkGVar : Names.identifier -> glob_constr
+val mkGApp : glob_constr*(glob_constr list) -> glob_constr
+val mkGLambda : Names.name * glob_constr * glob_constr -> glob_constr
+val mkGProd : Names.name * glob_constr * glob_constr -> glob_constr
+val mkGLetIn : Names.name * glob_constr * glob_constr -> glob_constr
+val mkGCases : glob_constr option * tomatch_tuples * cases_clauses -> glob_constr
+val mkGSort : glob_sort -> glob_constr
+val mkGHole : unit -> glob_constr (* we only build Evd.BinderType Anonymous holes *)
+val mkGCast : glob_constr* glob_constr -> glob_constr
(*
Some basic functions to decompose glob_constrs
These are analogous to the ones constrs