src/HOL/Library/Option_ord.thy
changeset 67091 1393c2340eec
parent 67006 b1278ed3cd46
child 67829 2a6ef5ba4822
--- a/src/HOL/Library/Option_ord.thy	Sun Nov 26 13:19:52 2017 +0100
+++ b/src/HOL/Library/Option_ord.thy	Sun Nov 26 21:08:32 2017 +0100
@@ -101,12 +101,12 @@
   fix z :: "'a option"
   assume H: "\<And>x. (\<And>y. y < x \<Longrightarrow> P y) \<Longrightarrow> P x"
   have "P None" by (rule H) simp
-  then have P_Some [case_names Some]: "P z" if "\<And>x. z = Some x \<Longrightarrow> (P o Some) x" for z
+  then have P_Some [case_names Some]: "P z" if "\<And>x. z = Some x \<Longrightarrow> (P \<circ> Some) x" for z
     using \<open>P None\<close> that by (cases z) simp_all
   show "P z"
   proof (cases z rule: P_Some)
     case (Some w)
-    show "(P o Some) w"
+    show "(P \<circ> Some) w"
     proof (induct rule: less_induct)
       case (less x)
       have "P (Some x)"
@@ -117,7 +117,7 @@
         proof (cases y rule: P_Some)
           case (Some v)
           with \<open>y < Some x\<close> have "v < x" by simp
-          with less show "(P o Some) v" .
+          with less show "(P \<circ> Some) v" .
         qed
       qed
       then show ?case by simp