eliminated obsolete C/flip combinator;
authorwenzelm
Wed, 14 Oct 2009 22:57:44 +0200
changeset 32934 a1b6e8d281ce
parent 32933 ba14400f7f34
child 32935 2218b970325a
eliminated obsolete C/flip combinator;
src/HOL/Library/normarith.ML
--- a/src/HOL/Library/normarith.ML	Wed Oct 14 21:14:53 2009 +0200
+++ b/src/HOL/Library/normarith.ML	Wed Oct 14 22:57:44 2009 +0200
@@ -347,7 +347,6 @@
  val concl = Thm.dest_arg o cprop_of
  fun conjunct1 th = th RS @{thm conjunct1}
  fun conjunct2 th = th RS @{thm conjunct2}
- fun C f x y = f y x
 fun real_vector_ineq_prover ctxt translator (ges,gts) = 
  let 
 (*   val _ = error "real_vector_ineq_prover: pause" *)
@@ -370,7 +369,7 @@
   val th11 = hd (Variable.export ctxt' ctxt [fold implies_intr shs th1])
   val cps = map (swap o Thm.dest_equals) (cprems_of th11)
   val th12 = instantiate ([], cps) th11
-  val th13 = fold (C implies_elim) (map (reflexive o snd) cps) th12;
+  val th13 = fold Thm.elim_implies (map (reflexive o snd) cps) th12;
  in hd (Variable.export ctxt' ctxt [th13])
  end 
 in val real_vector_ineq_prover = real_vector_ineq_prover