aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/LetPat.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/LetPat.v')
-rw-r--r--test-suite/success/LetPat.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/test-suite/success/LetPat.v b/test-suite/success/LetPat.v
index 72c7cc155..545b8aeb8 100644
--- a/test-suite/success/LetPat.v
+++ b/test-suite/success/LetPat.v
@@ -48,8 +48,8 @@ Definition identity_functor (c : category) : functor c c :=
fun x => x.
Definition functor_composition (a b c : category) : functor a b -> functor b c -> functor a c :=
- let ' (A :& homA :& CA) := a in
- let ' (B :& homB :& CB) := b in
- let ' (C :& homB :& CB) := c in
+ let 'A :& homA :& CA := a in
+ let 'B :& homB :& CB := b in
+ let 'C :& homB :& CB := c in
fun f g =>
- fun x : A => g (f x).
+ fun x => g (f x).