src/Pure/Isar/obtain.ML
changeset 60461 22995ec9fefd
parent 60456 323b15b5af73
child 60475 4c65bd64bba4
--- a/src/Pure/Isar/obtain.ML	Sat Jun 13 22:44:22 2015 +0200
+++ b/src/Pure/Isar/obtain.ML	Sat Jun 13 23:36:21 2015 +0200
@@ -158,8 +158,7 @@
       [(Binding.name Auto_Bind.thesisN, NONE, NoSyn)]
       (map (fn (a, A) => ((a, [Context_Rules.intro_query NONE]), [(A, [])])) obtains)
       [((Binding.empty, atts), [(thesis, [])])] int
-    |> (fn state' => state'
-        |> Proof.refine_insert (Assumption.local_prems_of (Proof.context_of state') ctxt))
+    |-> Proof.refine_insert
   end;
 
 in
@@ -233,8 +232,7 @@
       [(Binding.name Auto_Bind.thesisN, NONE, NoSyn)]
       [((that_binding, [Context_Rules.intro_query NONE]), [(that_prop, [])])]
       [(Thm.empty_binding, [(thesis, [])])] int
-    |> (fn state' => state'
-        |> Proof.refine_insert (Assumption.local_prems_of (Proof.context_of state') ctxt))
+    |-> Proof.refine_insert
     |> Proof.map_context (fold Variable.bind_term binds')
   end;
 
@@ -407,9 +405,12 @@
     |> Proof.fix [(Binding.name Auto_Bind.thesisN, NONE, NoSyn)]
     |> Proof.chain_facts chain_facts
     |> Proof.internal_goal print_result Proof_Context.mode_schematic "guess"
-      (SOME before_qed) after_qed [] [] [(Thm.empty_binding, [(Logic.mk_term goal, []), (goal, [])])]
+      (SOME before_qed) after_qed
+      [] [] [(Thm.empty_binding, [(Logic.mk_term goal, []), (goal, [])])]
+    |> snd
     |> Proof.refine (Method.primitive_text (fn _ => fn _ =>
-        Goal.init (Thm.cterm_of ctxt thesis))) |> Seq.hd
+        Goal.init (Thm.cterm_of ctxt thesis)))
+    |> Seq.hd
   end;
 
 in