src/HOL/Option.thy
changeset 55867 79b915f26533
parent 55531 601ca8efa000
child 57091 1fa9c19ba2c9
--- a/src/HOL/Option.thy	Mon Mar 03 12:48:20 2014 +0100
+++ b/src/HOL/Option.thy	Mon Mar 03 12:48:20 2014 +0100
@@ -28,7 +28,6 @@
 setup {* Sign.mandatory_path "option" *}
 
 lemmas inducts = option.induct
-lemmas recs = option.rec
 lemmas cases = option.case
 
 setup {* Sign.parent_path *}