aboutsummaryrefslogtreecommitdiff
path: root/spartan/lib/Maybe.thy
diff options
context:
space:
mode:
authorJosh Chen2020-07-08 15:55:48 +0200
committerJosh Chen2020-07-08 15:55:48 +0200
commit07c51b1801bd701bef61cedd571a944d9bd37e8b (patch)
tree16b9581f9f52af4058594cd503aa2eec1d2cb801 /spartan/lib/Maybe.thy
parentf0fab6e197510ce0e6d23a669f69de966701d495 (diff)
1. Initial `Definition` keyword. 2. ifelse.
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"