src/Pure/Isar/obtain.ML
changeset 50201 c26369c9eda6
parent 49660 de49d9b4d7bc
child 52456 960202346d0c
equal deleted inserted replaced
50200:2c94c065564e 50201:c26369c9eda6
   297         |> Proof.bind_terms Auto_Bind.no_facts
   297         |> Proof.bind_terms Auto_Bind.no_facts
   298       end;
   298       end;
   299 
   299 
   300     val goal = Var (("guess", 0), propT);
   300     val goal = Var (("guess", 0), propT);
   301     fun print_result ctxt' (k, [(s, [_, th])]) =
   301     fun print_result ctxt' (k, [(s, [_, th])]) =
   302       Proof_Display.print_results Isabelle_Markup.state int ctxt' (k, [(s, [th])]);
   302       Proof_Display.print_results Markup.state int ctxt' (k, [(s, [th])]);
   303     val before_qed = SOME (Method.primitive_text (Goal.conclude #> Raw_Simplifier.norm_hhf #>
   303     val before_qed = SOME (Method.primitive_text (Goal.conclude #> Raw_Simplifier.norm_hhf #>
   304         (fn th => Goal.protect (Conjunction.intr (Drule.mk_term (Thm.cprop_of th)) th))));
   304         (fn th => Goal.protect (Conjunction.intr (Drule.mk_term (Thm.cprop_of th)) th))));
   305     fun after_qed [[_, res]] =
   305     fun after_qed [[_, res]] =
   306       Proof.end_block #> guess_context (check_result ctxt thesis res);
   306       Proof.end_block #> guess_context (check_result ctxt thesis res);
   307   in
   307   in