changeset 613 | 018aabbffd08 |
parent 597 | 8a1c8dc72b5c |
--- a/Quot/Quotients.thy Mon Dec 07 23:45:51 2009 +0100 +++ b/Quot/Quotients.thy Tue Dec 08 01:00:21 2009 +0100 @@ -42,10 +42,6 @@ "sum_map f1 f2 (Inl a) = Inl (f1 a)" | "sum_map f1 f2 (Inr a) = Inr (f2 a)" - - - - fun noption_map::"('a \<Rightarrow> 'b) \<Rightarrow> ('a noption) \<Rightarrow> ('b noption)" where