changeset 618 | 8dfae5d97387 |
parent 613 | 018aabbffd08 |
--- a/Quot/Quotients.thy Tue Dec 08 11:17:56 2009 +0100 +++ b/Quot/Quotients.thy Tue Dec 08 11:20:01 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