aboutsummaryrefslogtreecommitdiff
path: root/spartan/data/Maybe.thy
diff options
context:
space:
mode:
Diffstat (limited to 'spartan/data/Maybe.thy')
-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)"