src/HOL/Tools/Sledgehammer/sledgehammer.ML
changeset 39008 83ca64a880ea
parent 39007 aae6a0d33c66
child 39009 a9a2efcaf721
equal deleted inserted replaced
39007:aae6a0d33c66 39008:83ca64a880ea
   175   Scan.this_string set_ClauseFormulaRelationN |-- $$ "("
   175   Scan.this_string set_ClauseFormulaRelationN |-- $$ "("
   176   |-- Scan.repeat parse_clause_formula_pair
   176   |-- Scan.repeat parse_clause_formula_pair
   177 val extract_clause_formula_relation =
   177 val extract_clause_formula_relation =
   178   Substring.full #> Substring.position set_ClauseFormulaRelationN
   178   Substring.full #> Substring.position set_ClauseFormulaRelationN
   179   #> snd #> Substring.position "." #> fst #> Substring.string
   179   #> snd #> Substring.position "." #> fst #> Substring.string
   180   #> explode #> filter_out (curry (op =) " ") #> parse_clause_formula_relation
   180   #> explode #> filter_out Symbol.is_blank #> parse_clause_formula_relation
   181   #> fst
   181   #> fst
   182 
   182 
   183 (* TODO: move to "Sledgehammer_Reconstruct" *)
   183 (* TODO: move to "Sledgehammer_Reconstruct" *)
   184 fun repair_conjecture_shape_and_theorem_names output conjecture_shape
   184 fun repair_conjecture_shape_and_theorem_names output conjecture_shape
   185                                               axiom_names =
   185                                               axiom_names =