src/HOL/Option.thy
changeset 31998 2c7a24f74db9
parent 31154 f919b8e67413
child 32069 6d28bbd33e2c
--- a/src/HOL/Option.thy	Tue Jul 14 10:53:44 2009 +0200
+++ b/src/HOL/Option.thy	Tue Jul 14 10:54:04 2009 +0200
@@ -94,7 +94,7 @@
 subsubsection {* Code generator setup *}
 
 definition is_none :: "'a option \<Rightarrow> bool" where
-  [code post]: "is_none x \<longleftrightarrow> x = None"
+  [code_post]: "is_none x \<longleftrightarrow> x = None"
 
 lemma is_none_code [code]:
   shows "is_none None \<longleftrightarrow> True"
@@ -105,7 +105,7 @@
   "is_none x \<longleftrightarrow> x = None"
   by (simp add: is_none_def)
 
-lemma [code inline]:
+lemma [code_inline]:
   "eq_class.eq x None \<longleftrightarrow> is_none x"
   by (simp add: eq is_none_none)