src/HOL/Library/Sum_of_Squares/sum_of_squares.ML
changeset 42616 92715b528e78
parent 41490 0f1e411a1448
child 44453 082edd97ffe1
equal deleted inserted replaced
42607:c8673078f915 42616:92715b528e78
     8 signature SUM_OF_SQUARES =
     8 signature SUM_OF_SQUARES =
     9 sig
     9 sig
    10   datatype proof_method = Certificate of RealArith.pss_tree | Prover of string -> string
    10   datatype proof_method = Certificate of RealArith.pss_tree | Prover of string -> string
    11   val sos_tac: (RealArith.pss_tree -> unit) -> proof_method -> Proof.context -> int -> tactic
    11   val sos_tac: (RealArith.pss_tree -> unit) -> proof_method -> Proof.context -> int -> tactic
    12   val trace: bool Config.T
    12   val trace: bool Config.T
    13   val setup: theory -> theory
       
    14   exception Failure of string;
    13   exception Failure of string;
    15 end
    14 end
    16 
    15 
    17 structure Sum_of_Squares: SUM_OF_SQUARES =
    16 structure Sum_of_Squares: SUM_OF_SQUARES =
    18 struct
    17 struct
    48 
    47 
    49 val abs_rat = Rat.abs;
    48 val abs_rat = Rat.abs;
    50 val pow2 = rat_pow rat_2;
    49 val pow2 = rat_pow rat_2;
    51 val pow10 = rat_pow rat_10;
    50 val pow10 = rat_pow rat_10;
    52 
    51 
    53 val (trace, setup_trace) = Attrib.config_bool "sos_trace" (K false);
    52 val trace = Attrib.setup_config_bool @{binding sos_trace} (K false);
    54 val setup = setup_trace;
       
    55 
    53 
    56 exception Sanity;
    54 exception Sanity;
    57 
    55 
    58 exception Unsolvable;
    56 exception Unsolvable;
    59 
    57