src/HOL/Multivariate_Analysis/normarith.ML
changeset 48112 b1240319ef15
parent 46497 89ccf66aa73d
child 51717 9e7d1c139569
equal deleted inserted replaced
48111:33414f2e82ab 48112:b1240319ef15
   374          (fold_rev (splitequation ctxt) eqs ges,gts), RealArith.Trivial)
   374          (fold_rev (splitequation ctxt) eqs ges,gts), RealArith.Trivial)
   375 end;
   375 end;
   376 
   376 
   377   fun init_conv ctxt =
   377   fun init_conv ctxt =
   378    Simplifier.rewrite (Simplifier.context ctxt
   378    Simplifier.rewrite (Simplifier.context ctxt
   379      (HOL_basic_ss addsimps ([(*@{thm vec_0}, @{thm vec_1},*) @{thm dist_norm}, @{thm diff_0_right}, @{thm right_minus}, @{thm diff_self}, @{thm norm_zero}] @ @{thms arithmetic_simps} @ @{thms norm_pths})))
   379      (HOL_basic_ss addsimps ([(*@{thm vec_0}, @{thm vec_1},*) @{thm dist_norm}, @{thm right_minus}, @{thm diff_self}, @{thm norm_zero}] @ @{thms arithmetic_simps} @ @{thms norm_pths})))
   380    then_conv Numeral_Simprocs.field_comp_conv
   380    then_conv Numeral_Simprocs.field_comp_conv
   381    then_conv nnf_conv
   381    then_conv nnf_conv
   382 
   382 
   383  fun pure ctxt = fst o RealArith.gen_prover_real_arith ctxt (real_vector_prover ctxt);
   383  fun pure ctxt = fst o RealArith.gen_prover_real_arith ctxt (real_vector_prover ctxt);
   384  fun norm_arith ctxt ct =
   384  fun norm_arith ctxt ct =