src/HOL/ex/Join_Theory.thy
changeset 77895 655bd3b0671b
parent 70525 1615b6808192
equal deleted inserted replaced
77894:186bd4012b78 77895:655bd3b0671b
    33 subsection \<open>Example application\<close>
    33 subsection \<open>Example application\<close>
    34 
    34 
    35 setup \<open>
    35 setup \<open>
    36   fn thy =>
    36   fn thy =>
    37     let val forked_thys = Par_List.map (fn i => Named_Target.theory_map (spec i) thy) (1 upto 10)
    37     let val forked_thys = Par_List.map (fn i => Named_Target.theory_map (spec i) thy) (1 upto 10)
    38     in Theory.join_theory forked_thys end
    38     in Context.join_thys forked_thys end
    39 \<close>
    39 \<close>
    40 
    40 
    41 term test1
    41 term test1
    42 thm test1
    42 thm test1
    43 
    43