equal
deleted
inserted
replaced
543 #2 oo Specification.theorems_cmd "" [(Binding.empty_atts, flat facts)] fixes)); |
543 #2 oo Specification.theorems_cmd "" [(Binding.empty_atts, flat facts)] fixes)); |
544 |
544 |
545 val _ = |
545 val _ = |
546 Outer_Syntax.local_theory \<^command_keyword>\<open>named_theorems\<close> |
546 Outer_Syntax.local_theory \<^command_keyword>\<open>named_theorems\<close> |
547 "declare named collection of theorems" |
547 "declare named collection of theorems" |
548 (Parse.and_list1 (Parse.binding -- Scan.optional Parse.text "" |
548 (Parse.and_list1 (Parse.binding -- Scan.optional Parse.text "") >> |
549 -- Scan.optional (\<^keyword>\<open>includes\<close> |-- Scan.repeat1 Parse.text) []) >> |
549 fold (fn (b, descr) => snd o Named_Theorems.declare b descr)); |
550 fold (fn ((b, descr), extends) => snd o Named_Theorems.declare b extends descr)); |
|
551 |
550 |
552 in end\<close> |
551 in end\<close> |
553 |
552 |
554 |
553 |
555 subsubsection \<open>Hide names\<close> |
554 subsubsection \<open>Hide names\<close> |