src/HOL/Option.thy
changeset 4133 0a08c2b9b1ed
parent 2019 b45d9f2042e0
child 4192 c38ab5af38b5
--- a/src/HOL/Option.thy	Tue Nov 04 20:47:38 1997 +0100
+++ b/src/HOL/Option.thy	Tue Nov 04 20:48:38 1997 +0100
@@ -7,5 +7,15 @@
 *)
 
 Option = Arith +
+
 datatype 'a option = None | Some 'a
+
+constdefs
+
+  the		:: "'a option => 'a"
+ "the Ú %y. case y of None => arbitrary | Some x => x"
+
+  option_map	:: "('a => 'b) => ('a option => 'b option)"
+ "option_map Ú %f y. case y of None => None | Some x => Some (f x)"
+
 end