aboutsummaryrefslogtreecommitdiff
path: root/spartan/lib/Maybe.thy
diff options
context:
space:
mode:
Diffstat (limited to 'spartan/lib/Maybe.thy')
-rw-r--r--spartan/lib/Maybe.thy6
1 files changed, 3 insertions, 3 deletions
diff --git a/spartan/lib/Maybe.thy b/spartan/lib/Maybe.thy
index 0a7ec21..da22a4e 100644
--- a/spartan/lib/Maybe.thy
+++ b/spartan/lib/Maybe.thy
@@ -25,10 +25,10 @@ Definition MaybeInd:
"\<And>a. a: A \<Longrightarrow> f a: C (some A a)"
"m: Maybe A"
shows "C m"
- using assms[unfolded Maybe_def none_def some_def]
+ using assms[unfolded Maybe_def none_def some_def, type]
apply (elim m)
- apply (rule \<open>_ \<Longrightarrow> _: C (inl _ _ _)\<close>)
- apply (elim, rule \<open>_: C (inr _ _ _)\<close>)
+ apply fact
+ apply (elim, fact)
done
Lemma Maybe_comp_none: