src/Provers/blast.ML
changeset 26939 1035c89b4c02
parent 26938 64e850c3da9e
child 27809 a1e409db516b
equal deleted inserted replaced
26938:64e850c3da9e 26939:1035c89b4c02
   612   | showTerm d (Abs(a,t))    = if d=0 then dummyVar
   612   | showTerm d (Abs(a,t))    = if d=0 then dummyVar
   613                                else Term.Abs(a, dummyT, showTerm (d-1) t)
   613                                else Term.Abs(a, dummyT, showTerm (d-1) t)
   614   | showTerm d (f $ u)       = if d=0 then dummyVar
   614   | showTerm d (f $ u)       = if d=0 then dummyVar
   615                                else Term.$ (showTerm d f, showTerm (d-1) u);
   615                                else Term.$ (showTerm d f, showTerm (d-1) u);
   616 
   616 
   617 fun string_of thy d t = Sign.string_of_term thy (showTerm d t);
   617 fun string_of thy d t = Syntax.string_of_term_global thy (showTerm d t);
   618 
   618 
   619 (*Convert a Goal to an ordinary Not.  Used also in dup_intr, where a goal like
   619 (*Convert a Goal to an ordinary Not.  Used also in dup_intr, where a goal like
   620   Ex(P) is duplicated as the assumption ~Ex(P). *)
   620   Ex(P) is duplicated as the assumption ~Ex(P). *)
   621 fun negOfGoal (Const ("*Goal*", _) $ G) = negate G
   621 fun negOfGoal (Const ("*Goal*", _) $ G) = negate G
   622   | negOfGoal G = G;
   622   | negOfGoal G = G;
   636   let val t' = norm (negOfGoal t)
   636   let val t' = norm (negOfGoal t)
   637       val stm = string_of thy 8 t'
   637       val stm = string_of thy 8 t'
   638   in
   638   in
   639       case topType thy t' of
   639       case topType thy t' of
   640           NONE   => stm   (*no type to attach*)
   640           NONE   => stm   (*no type to attach*)
   641         | SOME T => stm ^ "\t:: " ^ Sign.string_of_typ thy T
   641         | SOME T => stm ^ "\t:: " ^ Syntax.string_of_typ_global thy T
   642   end;
   642   end;
   643 
   643 
   644 
   644 
   645 (*Print tracing information at each iteration of prover*)
   645 (*Print tracing information at each iteration of prover*)
   646 fun tracing (State {thy, fullTrace, ...}) brs =
   646 fun tracing (State {thy, fullTrace, ...}) brs =