src/Pure/more_thm.ML
changeset 49058 2924a83a4a0b
parent 49011 9c68e43502ce
child 49062 7e31dfd99ce7
equal deleted inserted replaced
49042:01041f7bf9b4 49058:2924a83a4a0b
    94   val corollaryK: string
    94   val corollaryK: string
    95   val legacy_get_kind: thm -> string
    95   val legacy_get_kind: thm -> string
    96   val kind_rule: string -> thm -> thm
    96   val kind_rule: string -> thm -> thm
    97   val kind: string -> attribute
    97   val kind: string -> attribute
    98   val register_proofs: thm list -> Context.generic -> Context.generic
    98   val register_proofs: thm list -> Context.generic -> Context.generic
       
    99   val register_proofs_thy: thm list -> theory -> theory
    99   val begin_proofs: Context.generic -> Context.generic
   100   val begin_proofs: Context.generic -> Context.generic
   100   val join_local_proofs: Proof.context -> unit
   101   val join_local_proofs: Proof.context -> unit
   101   val join_recent_proofs: theory -> unit
   102   val join_recent_proofs: theory -> unit
   102   val join_theory_proofs: theory -> unit
   103   val join_theory_proofs: theory -> unit
   103 end;
   104 end;
   491   fun merge _ = empty;
   492   fun merge _ = empty;
   492 );
   493 );
   493 
   494 
   494 val begin_proofs = Proofs.map (apfst (K empty_proofs));
   495 val begin_proofs = Proofs.map (apfst (K empty_proofs));
   495 val register_proofs = Proofs.map o pairself o add_proofs;
   496 val register_proofs = Proofs.map o pairself o add_proofs;
       
   497 val register_proofs_thy = Context.theory_map o register_proofs;
   496 
   498 
   497 val join_local_proofs = force_proofs o #1 o Proofs.get o Context.Proof;
   499 val join_local_proofs = force_proofs o #1 o Proofs.get o Context.Proof;
   498 val join_recent_proofs = force_proofs o #1 o Proofs.get o Context.Theory;
   500 val join_recent_proofs = force_proofs o #1 o Proofs.get o Context.Theory;
   499 val join_theory_proofs = force_proofs o #2 o Proofs.get o Context.Theory;
   501 val join_theory_proofs = force_proofs o #2 o Proofs.get o Context.Theory;
   500 
   502