doc-src/TutorialI/Types/Typedefs.thy
changeset 11901 e1aa90e4ef4e
parent 11858 ca128c9100b6
child 12332 aea72a834c85
equal deleted inserted replaced
11900:f8f37d61fbc2 11901:e1aa90e4ef4e
   201 @{thm[display]le_SucE}
   201 @{thm[display]le_SucE}
   202 reduces @{prop"n\<le>2"} to the three cases @{prop"n\<le>0"}, @{prop"n=1"} and
   202 reduces @{prop"n\<le>2"} to the three cases @{prop"n\<le>0"}, @{prop"n=1"} and
   203 @{prop"n=2"} which are trivial for simplification:
   203 @{prop"n=2"} which are trivial for simplification:
   204 *}
   204 *}
   205 
   205 
   206 apply(simp add: three_def numerals)
   206 apply(simp add: three_def numerals)   (* FIXME !? *)
   207 apply((erule le_SucE)+)
   207 apply((erule le_SucE)+)
   208 apply simp_all
   208 apply simp_all
   209 done
   209 done
   210 
   210 
   211 text{*
   211 text{*