src/HOL/Mutabelle/mutabelle.ML
changeset 41408 08a072ca6348
parent 41067 c78a2d402736
child 41755 404d94506599
equal deleted inserted replaced
41407:2878845bc549 41408:08a072ca6348
     1 (*  Title:      HOL/Mutabelle/mutabelle.ML
     1 (*  Title:      HOL/Mutabelle/mutabelle.ML
     2     Author:     Veronika Ortner, TU Muenchen
     2     Author:     Veronika Ortner, TU Muenchen
     3 
     3 
     4     Mutation of theorems
     4 Mutation of theorems.
     5 *)
     5 *)
       
     6 
     6 signature MUTABELLE =
     7 signature MUTABELLE =
     7 sig
     8 sig
     8  val testgen_name : string Unsynchronized.ref
     9  val testgen_name : string Unsynchronized.ref
     9  exception WrongPath of string;
    10  exception WrongPath of string;
    10  exception WrongArg of string;
    11  exception WrongArg of string;
    78    List.mapPartial (fn (s, (T, NONE)) => SOME (s, T) | _ => NONE)
    79    List.mapPartial (fn (s, (T, NONE)) => SOME (s, T) | _ => NONE)
    79      (filter_out (fn (s, _) => Name_Space.is_concealed namespace s) consts)
    80      (filter_out (fn (s, _) => Name_Space.is_concealed namespace s) consts)
    80  end;
    81  end;
    81 
    82 
    82 
    83 
    83 (*helper function in order to properly print a term*)
    84 (*possibility to print a given term for debugging purposes*)
    84 
    85 
    85 fun prt x = Pretty.writeln (Syntax.pretty_term_global @{theory Main} x);
    86 fun prt x = Pretty.writeln (Syntax.pretty_term_global @{theory Main} x);
    86 
       
    87 
       
    88 (*possibility to print a given term for debugging purposes*)
       
    89 
    87 
    90 val debug = (Unsynchronized.ref false);
    88 val debug = (Unsynchronized.ref false);
    91 fun debug_msg mutterm = if (!debug) then (prt mutterm) else ();
    89 fun debug_msg mutterm = if (!debug) then (prt mutterm) else ();
    92 
    90 
    93 
    91