aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/Cases.out
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-10-20 12:56:43 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-10-20 23:29:19 +0200
commit7efeff178470ab204e531cd07176091bf5022da6 (patch)
treeafdc79d6eb2a371fa2cec235aabea3c5425d46b9 /test-suite/output/Cases.out
parentf00f8482e1d21ef8b03044ed2162cb29d9e4537d (diff)
A patch for printing "match" when constructors are defined with let-in
but the internal representation dropped let-in. Ideally, the internal representation of the "match" should use contexts for the predicate and the branches. This would however be a rather significant change. In the meantime, just a hack. To do, there is still an extra @ in the constructor name that does not need to be there.
Diffstat (limited to 'test-suite/output/Cases.out')
-rw-r--r--test-suite/output/Cases.out8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/output/Cases.out b/test-suite/output/Cases.out
index c768f09ce..0ebc251bc 100644
--- a/test-suite/output/Cases.out
+++ b/test-suite/output/Cases.out
@@ -8,6 +8,14 @@ fix F (t : t) : P t :=
(let x := t in forall x0 : x, P x0 -> P (k x0)) -> forall t : t, P t
t_rect is not universe polymorphic
+ = fun d : A => match d with
+ | @C _ _ b => b
+ end
+ : A -> 0 = 0
+ = fun d : A => match d with
+ | @C _ _ b => b
+ end
+ : A -> 0 = 0
proj =
fun (x y : nat) (P : nat -> Type) (def : P x) (prf : P y) =>
match Nat.eq_dec x y with