aboutsummaryrefslogtreecommitdiff
path: root/spartan/lib/List.thy
diff options
context:
space:
mode:
Diffstat (limited to 'spartan/lib/List.thy')
-rw-r--r--spartan/lib/List.thy2
1 files changed, 1 insertions, 1 deletions
diff --git a/spartan/lib/List.thy b/spartan/lib/List.thy
index dd51582..83e5149 100644
--- a/spartan/lib/List.thy
+++ b/spartan/lib/List.thy
@@ -149,7 +149,7 @@ Definition map:
proof (elim xs)
show "[]: List B" by intro
next fix x ys
- assume "x: A" "ys: List B"
+ assuming "x: A" "ys: List B"
show "f x # ys: List B" by typechk
qed