src/Pure/Isar/obtain.ML
changeset 33386 ff29d1549aca
parent 33369 470a7b233ee5
child 33389 bb3a5fa94a91
--- a/src/Pure/Isar/obtain.ML	Mon Nov 02 20:38:46 2009 +0100
+++ b/src/Pure/Isar/obtain.ML	Mon Nov 02 20:45:23 2009 +0100
@@ -129,7 +129,7 @@
     val _ = Variable.warn_extra_tfrees fix_ctxt asms_ctxt;
 
     (*obtain statements*)
-    val thesisN = Name.variant xs AutoBind.thesisN;
+    val thesisN = Name.variant xs Auto_Bind.thesisN;
     val (thesis_var, thesis) = #1 (bind_judgment fix_ctxt thesisN);
 
     val asm_frees = fold Term.add_frees asm_props [];
@@ -142,7 +142,7 @@
       Term.list_all_free (parms, Logic.list_implies (asm_props, thesis))
       |> Library.curry Logic.list_rename_params xs;
     val obtain_prop =
-      Logic.list_rename_params ([AutoBind.thesisN],
+      Logic.list_rename_params ([Auto_Bind.thesisN],
         Term.list_all_free ([thesis_var], Logic.mk_implies (that_prop, thesis)));
 
     fun after_qed _ =
@@ -189,7 +189,7 @@
     val thy = ProofContext.theory_of ctxt;
     val cert = Thm.cterm_of thy;
 
-    val ((thesis_var, thesis), thesis_ctxt) = bind_judgment ctxt AutoBind.thesisN;
+    val ((thesis_var, thesis), thesis_ctxt) = bind_judgment ctxt Auto_Bind.thesisN;
     val rule =
       (case SINGLE (Method.insert_tac facts 1 THEN tac thesis_ctxt) (Goal.init (cert thesis)) of
         NONE => raise THM ("Obtain.result: tactic failed", 0, facts)
@@ -273,7 +273,7 @@
     val ctxt = Proof.context_of state;
     val chain_facts = if can Proof.assert_chain state then Proof.the_facts state else [];
 
-    val (thesis_var, thesis) = #1 (bind_judgment ctxt AutoBind.thesisN);
+    val (thesis_var, thesis) = #1 (bind_judgment ctxt Auto_Bind.thesisN);
     val vars = ctxt |> prep_vars raw_vars |-> fold_map inferred_type |> fst |> polymorphic ctxt;
 
     fun guess_context raw_rule state' =
@@ -293,7 +293,7 @@
         |> Proof.fix_i (map (fn ((x, T), mx) => (Binding.name x, SOME T, mx)) parms)
         |> `Proof.context_of |-> (fn fix_ctxt => Proof.assm_i
           (obtain_export fix_ctxt rule (map cert ts)) [(Thm.empty_binding, asms)])
-        |> Proof.bind_terms AutoBind.no_facts
+        |> Proof.bind_terms Auto_Bind.no_facts
       end;
 
     val goal = Var (("guess", 0), propT);
@@ -307,7 +307,7 @@
     state
     |> Proof.enter_forward
     |> Proof.begin_block
-    |> Proof.fix_i [(Binding.name AutoBind.thesisN, NONE, NoSyn)]
+    |> Proof.fix_i [(Binding.name Auto_Bind.thesisN, NONE, NoSyn)]
     |> Proof.chain_facts chain_facts
     |> Proof.local_goal print_result (K I) (apsnd (rpair I))
       "guess" before_qed after_qed [(Thm.empty_binding, [Logic.mk_term goal, goal])]