src/Doc/Eisbach/Manual.thy
changeset 61853 fb7756087101
parent 61656 cfabbc083977
child 61912 ad710de5c576
equal deleted inserted replaced
61852:d273c24b5776 61853:fb7756087101
   929   auxiliary function.
   929   auxiliary function.
   930 \<close>
   930 \<close>
   931 
   931 
   932     attribute_setup get_split_rule =
   932     attribute_setup get_split_rule =
   933       \<open>Args.term >> (fn t =>
   933       \<open>Args.term >> (fn t =>
   934         Thm.rule_attribute (fn context => fn _ =>
   934         Thm.rule_attribute [] (fn context => fn _ =>
   935           (case get_split_rule (Context.proof_of context) t of
   935           (case get_split_rule (Context.proof_of context) t of
   936             SOME thm => thm
   936             SOME thm => thm
   937           | NONE => Drule.dummy_thm)))\<close>
   937           | NONE => Drule.dummy_thm)))\<close>
   938 
   938 
   939 text \<open>
   939 text \<open>