src/HOL/Tools/Metis/metis_tactic.ML
changeset 70514 7a63b16c53c4
parent 70513 dc749e0dc6b2
child 73932 fd21b4a93043
equal deleted inserted replaced
70513:dc749e0dc6b2 70514:7a63b16c53c4
   174     fun get_isa_thm mth Isa_Reflexive_or_Trivial =
   174     fun get_isa_thm mth Isa_Reflexive_or_Trivial =
   175           reflexive_or_trivial_of_metis ctxt type_enc sym_tab concealed mth
   175           reflexive_or_trivial_of_metis ctxt type_enc sym_tab concealed mth
   176       | get_isa_thm mth Isa_Lambda_Lifted =
   176       | get_isa_thm mth Isa_Lambda_Lifted =
   177           lam_lifted_of_metis ctxt type_enc sym_tab concealed mth
   177           lam_lifted_of_metis ctxt type_enc sym_tab concealed mth
   178       | get_isa_thm _ (Isa_Raw ith) = ith
   178       | get_isa_thm _ (Isa_Raw ith) = ith
   179     val axioms = axioms |> map (fn (mth, ith) => (mth, get_isa_thm mth ith))
   179     val axioms = axioms |> map (fn (mth, ith) =>
       
   180       (mth, get_isa_thm mth ith |> Thm.close_derivation \<^here>))
   180     val _ = trace_msg ctxt (K "ISABELLE CLAUSES")
   181     val _ = trace_msg ctxt (K "ISABELLE CLAUSES")
   181     val _ = List.app (fn (_, ith) => trace_msg ctxt (fn () => Thm.string_of_thm ctxt ith)) axioms
   182     val _ = List.app (fn (_, ith) => trace_msg ctxt (fn () => Thm.string_of_thm ctxt ith)) axioms
   182     val _ = trace_msg ctxt (K "METIS CLAUSES")
   183     val _ = trace_msg ctxt (K "METIS CLAUSES")
   183     val _ = List.app (fn (mth, _) => trace_msg ctxt (fn () => Metis_Thm.toString mth)) axioms
   184     val _ = List.app (fn (mth, _) => trace_msg ctxt (fn () => Metis_Thm.toString mth)) axioms
   184 
   185