src/Pure/Isar/class_target.ML
changeset 36323 655e2d74de3a
parent 36106 19deea200358
child 36328 4d9deabf6474
equal deleted inserted replaced
36322:81cba3921ba5 36323:655e2d74de3a
   368     fun after_qed results =
   368     fun after_qed results =
   369       ProofContext.theory ((fold o fold) AxClass.add_classrel results);
   369       ProofContext.theory ((fold o fold) AxClass.add_classrel results);
   370   in
   370   in
   371     thy
   371     thy
   372     |> ProofContext.init
   372     |> ProofContext.init
   373     |> Proof.theorem_i NONE after_qed [[(mk_prop thy classrel, [])]]
   373     |> Proof.theorem NONE after_qed [[(mk_prop thy classrel, [])]]
   374   end;
   374   end;
   375 
   375 
   376 in
   376 in
   377 
   377 
   378 val classrel =
   378 val classrel =
   537     lthy
   537     lthy
   538     |> do_proof after_qed' arities_proof
   538     |> do_proof after_qed' arities_proof
   539   end;
   539   end;
   540 
   540 
   541 val instantiation_instance = gen_instantiation_instance (fn after_qed => fn ts =>
   541 val instantiation_instance = gen_instantiation_instance (fn after_qed => fn ts =>
   542   Proof.theorem_i NONE (after_qed o map the_single) (map (fn t => [(t, [])]) ts));
   542   Proof.theorem NONE (after_qed o map the_single) (map (fn t => [(t, [])]) ts));
   543 
   543 
   544 fun prove_instantiation_instance tac = gen_instantiation_instance (fn after_qed =>
   544 fun prove_instantiation_instance tac = gen_instantiation_instance (fn after_qed =>
   545   fn ts => fn lthy => after_qed (map (fn t => Goal.prove lthy [] [] t
   545   fn ts => fn lthy => after_qed (map (fn t => Goal.prove lthy [] [] t
   546     (fn {context, ...} => tac context)) ts) lthy) I;
   546     (fn {context, ...} => tac context)) ts) lthy) I;
   547 
   547 
   593     fun after_qed results = ProofContext.theory
   593     fun after_qed results = ProofContext.theory
   594       ((fold o fold) AxClass.add_arity results);
   594       ((fold o fold) AxClass.add_arity results);
   595   in
   595   in
   596     thy
   596     thy
   597     |> ProofContext.init
   597     |> ProofContext.init
   598     |> Proof.theorem_i NONE after_qed (map (fn t => [(t, [])]) arities)
   598     |> Proof.theorem NONE after_qed (map (fn t => [(t, [])]) arities)
   599   end;
   599   end;
   600 
   600 
   601 
   601 
   602 (** tactics and methods **)
   602 (** tactics and methods **)
   603 
   603