src/HOL/Tools/Sledgehammer/sledgehammer_hol_clause.ML
changeset 37515 ef3742657bc6
parent 37512 ff72d3ddc898
child 37566 9ca40dff25bd
equal deleted inserted replaced
37514:b147d01b8ebc 37515:ef3742657bc6
   214   let
   214   let
   215     val (skolem_somes, cls) = make_clause thy (id, name, Axiom, th) skolem_somes
   215     val (skolem_somes, cls) = make_clause thy (id, name, Axiom, th) skolem_somes
   216   in (skolem_somes, clss |> not (isTaut cls) ? cons (name, cls)) end
   216   in (skolem_somes, clss |> not (isTaut cls) ? cons (name, cls)) end
   217 
   217 
   218 fun make_axiom_clauses thy clauses =
   218 fun make_axiom_clauses thy clauses =
   219   ([], []) |> fold (add_axiom_clause thy) clauses |> snd
   219   ([], []) |> fold_rev (add_axiom_clause thy) clauses |> snd
   220 
   220 
   221 fun make_conjecture_clauses thy =
   221 fun make_conjecture_clauses thy =
   222   let
   222   let
   223     fun aux _ _ [] = []
   223     fun aux _ _ [] = []
   224       | aux n skolem_somes (th :: ths) =
   224       | aux n skolem_somes (th :: ths) =