src/Pure/Pure.thy
changeset 70182 ca9dfa7ee3bd
parent 70177 b67bab2b132c
child 70205 3293471cf176
--- a/src/Pure/Pure.thy	Thu Apr 18 06:19:30 2019 +0200
+++ b/src/Pure/Pure.thy	Wed Apr 17 16:57:06 2019 +0000
@@ -545,9 +545,8 @@
 val _ =
   Outer_Syntax.local_theory \<^command_keyword>\<open>named_theorems\<close>
     "declare named collection of theorems"
-    (Parse.and_list1 (Parse.binding -- Scan.optional Parse.text ""
-      -- Scan.optional (\<^keyword>\<open>includes\<close> |-- Scan.repeat1 Parse.text) []) >>
-      fold (fn ((b, descr), extends) => snd o Named_Theorems.declare b extends descr));
+    (Parse.and_list1 (Parse.binding -- Scan.optional Parse.text "") >>
+      fold (fn (b, descr) => snd o Named_Theorems.declare b descr));
 
 in end\<close>