order conjunctions to be printed without parentheses
authorhoelzl
Tue, 13 Oct 2009 13:40:26 +0200
changeset 32920 ccfb774af58c
parent 32919 37adfa07b54b
child 32923 0b92e6359bc4
order conjunctions to be printed without parentheses
src/HOL/Decision_Procs/Approximation.thy
--- a/src/HOL/Decision_Procs/Approximation.thy	Tue Oct 13 12:02:55 2009 +0200
+++ b/src/HOL/Decision_Procs/Approximation.thy	Tue Oct 13 13:40:26 2009 +0200
@@ -3473,7 +3473,7 @@
        |> HOLogic.dest_list
        |> curry ListPair.zip (HOLogic.dest_list xs @ calculated_subterms arith_term)
        |> map (fn (elem, s) => @{term "op : :: real \<Rightarrow> real set \<Rightarrow> bool"} $ elem $ mk_result prec (dest_ivl s))
-       |> foldl1 HOLogic.mk_conj))
+       |> foldr1 HOLogic.mk_conj))
 
   fun approx_arith prec ctxt t = realify t
        |> Reflection.genreif ctxt form_equations