aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Case13.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-11 12:40:31 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-10-11 12:45:52 +0200
commitaf3538f0c6decdccd47abcdeb7b7eeaff64b69b5 (patch)
tree245ee69c69f10e9e2da36b14ee3a832e2f5cf456 /test-suite/success/Case13.v
parente3798c52c3bd52d43fa84feedd7caaa4def57db8 (diff)
Reverting generalization and cleaning of the return clause inference in v8.6.
The move to systematically trying small inversion first bumps sometimes as feared to the weakness of unification (see #5107). ---- Revert "Posssible abstractions over goal variables when inferring match return clause." This reverts commit 0658ba7b908dad946200f872f44260d0e4893a94. Revert "Trying an abstracting dependencies heuristic for the match return clause even when no type constraint is given." This reverts commit 292f365185b7acdee79f3ff7b158551c2764c548. Revert "Trying a no-inversion no-dependency heuristic for match return clause." This reverts commit 2422aeb2b59229891508f35890653a9737988c00.
Diffstat (limited to 'test-suite/success/Case13.v')
-rw-r--r--test-suite/success/Case13.v38
1 files changed, 0 insertions, 38 deletions
diff --git a/test-suite/success/Case13.v b/test-suite/success/Case13.v
index 356a67efe..8f95484cf 100644
--- a/test-suite/success/Case13.v
+++ b/test-suite/success/Case13.v
@@ -87,41 +87,3 @@ Check fun (x : E) => match x with c => e c end.
Inductive C' : bool -> Set := c' : C' true.
Inductive E' (b : bool) : Set := e' :> C' b -> E' b.
Check fun (x : E' true) => match x with c' => e' true c' end.
-
-(* Check use of the no-dependency strategy when a type constraint is
- given (and when the "inversion-and-dependencies-as-evars" strategy
- is not strong enough because of a constructor with a type whose
- pattern structure is not refined enough for it to be captured by
- the inversion predicate) *)
-
-Inductive K : bool -> bool -> Type := F : K true true | G x : K x x.
-
-Check fun z P Q (y:K true z) (H1 H2:P y) (f:forall y, P y -> Q y z) =>
- match y with
- | F => f y H1
- | G _ => f y H2
- end : Q y z.
-
-(* Check use of the maximal-dependency-in-variable strategy even when
- no explicit type constraint is given (and when the
- "inversion-and-dependencies-as-evars" strategy is not strong enough
- because of a constructor with a type whose pattern structure is not
- refined enough for it to be captured by the inversion predicate) *)
-
-Check fun z P Q (y:K true z) (H1 H2:P y) (f:forall y z, P y -> Q y z) =>
- match y with
- | F => f y true H1
- | G b => f y b H2
- end.
-
-(* Check use of the maximal-dependency-in-variable strategy for "Var"
- variables *)
-
-Goal forall z P Q (y:K true z) (H1 H2:P y) (f:forall y z, P y -> Q y z), Q y z.
-intros z P Q y H1 H2 f.
-Show.
-refine (match y with
- | F => f y true H1
- | G b => f y b H2
- end).
-Qed.