src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML
changeset 36491 6769f8eacaac
parent 36476 a04cf4704668
child 36493 a3357a631b96
equal deleted inserted replaced
36490:5abf45444a16 36491:6769f8eacaac
   183 
   183 
   184 fun make_schematic_type_var (x,i) =
   184 fun make_schematic_type_var (x,i) =
   185       tvar_prefix ^ (ascii_of_indexname (trim_type_var x,i));
   185       tvar_prefix ^ (ascii_of_indexname (trim_type_var x,i));
   186 fun make_fixed_type_var x = tfree_prefix ^ (ascii_of (trim_type_var x));
   186 fun make_fixed_type_var x = tfree_prefix ^ (ascii_of (trim_type_var x));
   187 
   187 
   188 val max_dfg_symbol_length = 63
   188 val max_dfg_symbol_length =
       
   189   if is_new_spass_version then 1000000 (* arbitrary large number *) else 63
   189 
   190 
   190 (* HACK because SPASS 3.0 truncates identifiers to 63 characters. *)
   191 (* HACK because SPASS 3.0 truncates identifiers to 63 characters. *)
   191 fun controlled_length dfg s =
   192 fun controlled_length dfg s =
   192   if dfg andalso size s > max_dfg_symbol_length then
   193   if dfg andalso size s > max_dfg_symbol_length then
   193     String.extract (s, 0, SOME (max_dfg_symbol_length div 2 - 1)) ^ "__" ^
   194     String.extract (s, 0, SOME (max_dfg_symbol_length div 2 - 1)) ^ "__" ^