src/Pure/ex/Guess.thy
changeset 82317 231b6d8231c6
parent 82048 2ea9f9ed19c6
child 82643 f1c14af17591
equal deleted inserted replaced
82316:83584916b6d7 82317:231b6d8231c6
   145         |> Proof.map_context (fold Variable.unbind_term Auto_Bind.no_facts)
   145         |> Proof.map_context (fold Variable.unbind_term Auto_Bind.no_facts)
   146       end;
   146       end;
   147 
   147 
   148     val guess = (("guess", 0), propT);
   148     val guess = (("guess", 0), propT);
   149     val goal = Var guess;
   149     val goal = Var guess;
   150     val pos = Position.thread_data ();
       
   151     fun print_result ctxt' (k, [(s, [_, th])]) =
   150     fun print_result ctxt' (k, [(s, [_, th])]) =
   152       Proof_Display.print_results {interactive = int, pos = pos, proof_state = true}
   151       Proof_Display.print_results {interactive = int, pos = Position.thread_data ()}
   153         ctxt' (k, [(s, [th])]);
   152         ctxt' (k, [(s, [th])]);
   154     val before_qed =
   153     val before_qed =
   155       Method.primitive_text (fn ctxt =>
   154       Method.primitive_text (fn ctxt =>
   156         Goal.conclude #> Raw_Simplifier.norm_hhf ctxt #>
   155         Goal.conclude #> Raw_Simplifier.norm_hhf ctxt #>
   157           (fn th => Goal.protect 0 (Conjunction.intr (Drule.mk_term (Thm.cprop_of th)) th)));
   156           (fn th => Goal.protect 0 (Conjunction.intr (Drule.mk_term (Thm.cprop_of th)) th)));