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.thy2
1 files changed, 1 insertions, 1 deletions
diff --git a/spartan/lib/Maybe.thy b/spartan/lib/Maybe.thy
index 1efbb95..6729812 100644
--- a/spartan/lib/Maybe.thy
+++ b/spartan/lib/Maybe.thy
@@ -17,7 +17,7 @@ lemma
Maybe_some: "a: A \<Longrightarrow> some A a: Maybe A"
unfolding Maybe_def none_def some_def by typechk+
-Lemma (derive) MaybeInd:
+Definition MaybeInd:
assumes
"A: U i"
"\<And>m. m: Maybe A \<Longrightarrow> C m: U i"