aboutsummaryrefslogtreecommitdiff
path: root/src/Reflection/InputSyntax.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2016-09-05 14:31:23 -0700
committerGravatar Jason Gross <jagro@google.com>2016-09-05 15:31:28 -0700
commitf789524d8e0542d8ff9ff1357ffa2261509c7bfa (patch)
treeeebc6ff48f2ad606dfa3b14537185c1327ea8682 /src/Reflection/InputSyntax.v
parent71253e65b115f6332c544476bfe680a8d3f18568 (diff)
More 8.4 fixes
Diffstat (limited to 'src/Reflection/InputSyntax.v')
-rw-r--r--src/Reflection/InputSyntax.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/src/Reflection/InputSyntax.v b/src/Reflection/InputSyntax.v
index fda06683a..c3c796d75 100644
--- a/src/Reflection/InputSyntax.v
+++ b/src/Reflection/InputSyntax.v
@@ -36,7 +36,7 @@ Section language.
| MatchPair : forall {t1 t2}, exprf (Prod t1 t2) -> forall {tC}, (var t1 -> var t2 -> exprf tC) -> exprf tC.
Inductive expr : type -> Type :=
| Return {t} : exprf t -> expr t
- | Abs {src dst} : (var (Tbase src) -> expr dst) -> expr (src -> dst).
+ | Abs {src dst} : (var (Tbase src) -> expr dst) -> expr (Arrow src dst).
Global Coercion Return : exprf >-> expr.
End expr.
@@ -111,7 +111,7 @@ Section language.
pose (e (interp_flat_type_gen interp_base_type)) as E.
repeat match goal with |- context[e ?f] => change (e f) with E end.
refine match E with
- | Abs _ _ _ => idProp (* small inversions *)
+ | Abs _ _ _ => fun x : Prop => x (* small inversions *)
| Return _ _ => _
end.
apply compilef_correct.