diff options
| author | pboutill | 2010-05-18 15:57:18 +0000 |
|---|---|---|
| committer | pboutill | 2010-05-18 15:57:18 +0000 |
| commit | e7c9f5f130f5187e5d9b43c8f0ed15deb49e4b2c (patch) | |
| tree | 970e35349cfa40f40c51ba5089073210d450df51 /kernel/declarations.ml | |
| parent | 6cca4015db457f91b8eb9cf824f21246cbe7c6e6 (diff) | |
Applicative commutative cuts in Fixpoint guard condition
In "(match ... with |... -> fun x -> t end) u", "x" has now the subterm
property of "u" in the analysis of "t".
Commutative cuts aren't compatible with typing so we need to ensure that
term of "x"'s type and term of "u"'s have the same subterm_spec.
Consequently,declaration.MRec argument has changed to the inductive name
instead of only the number of the inductive in the mutual_inductive
family.
In subterm_specif and check_rec_call, arguments are stored in a stack.
At each lambda, one element is popped to add in renv a smarter
subterm_spec for the variable. subterm_spec of constructor's argument
was added this way, the job is now done more often.
Some eta contracted match branches are now accepted but enforcing
eta-expansion of branches might be anyway a recommended invariant.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13012 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/declarations.ml')
| -rw-r--r-- | kernel/declarations.ml | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/kernel/declarations.ml b/kernel/declarations.ml index 4f98bb8b07..c7f8087428 100644 --- a/kernel/declarations.ml +++ b/kernel/declarations.ml @@ -71,7 +71,7 @@ let subst_rel_context sub = list_smartmap (subst_rel_declaration sub) type recarg = | Norec - | Mrec of int + | Mrec of inductive | Imbr of inductive let subst_recarg sub r = match r with |
