aboutsummaryrefslogtreecommitdiff
path: root/spartan/data/Maybe.thy
diff options
context:
space:
mode:
authorJosh Chen2020-05-28 14:08:26 +0200
committerJosh Chen2020-05-28 14:08:26 +0200
commit1ccd93665a01acdc25b37409e94b71615ced5393 (patch)
tree450284e77c40512408b0849f3ca2b12367aa4b90 /spartan/data/Maybe.thy
parent6ff59c83de9ce7d5715fae19f50d94b0b973414a (diff)
more List and Maybe
Diffstat (limited to '')
-rw-r--r--spartan/data/Maybe.thy6
1 files changed, 4 insertions, 2 deletions
diff --git a/spartan/data/Maybe.thy b/spartan/data/Maybe.thy
index 98f5283..1efbb95 100644
--- a/spartan/data/Maybe.thy
+++ b/spartan/data/Maybe.thy
@@ -55,8 +55,10 @@ Lemma Maybe_comp_some:
lemmas
[intros] = MaybeF Maybe_none Maybe_some and
- MaybeE [elims "?m"] = MaybeInd and
- [comps] = Maybe_comp_none Maybe_comp_some
+ [comps] = Maybe_comp_none Maybe_comp_some and
+ MaybeE [elims "?m"] = MaybeInd[rotated 4]
+lemmas
+ Maybe_cases [cases] = MaybeE
abbreviation "MaybeRec A C \<equiv> MaybeInd A (K C)"