src/Pure/tctical.ML
changeset 10767 8fa4aafa7314
parent 8535 7428194b39f7
child 10821 dcb75538f542
equal deleted inserted replaced
10766:ace2ba2d4fd1 10767:8fa4aafa7314
   372   to avoid copying.  Proof states have X==concl as an assuption.*)
   372   to avoid copying.  Proof states have X==concl as an assuption.*)
   373 
   373 
   374 val prop_equals = cterm_of (Theory.sign_of ProtoPure.thy) 
   374 val prop_equals = cterm_of (Theory.sign_of ProtoPure.thy) 
   375                     (Const("==", propT-->propT-->propT));
   375                     (Const("==", propT-->propT-->propT));
   376 
   376 
   377 fun mk_prop_equals(t,u) = capply (capply prop_equals t) u;
   377 fun mk_prop_equals(t,u) = Thm.capply (Thm.capply prop_equals t) u;
   378 
   378 
   379 (*Like trivial but returns [ct==X] ct==>X instead of ct==>ct, if possible.
   379 (*Like trivial but returns [ct==X] ct==>X instead of ct==>ct, if possible.
   380   It is paired with a function to undo the transformation.  If ct contains
   380   It is paired with a function to undo the transformation.  If ct contains
   381   Vars then it returns ct==>ct.*)
   381   Vars then it returns ct==>ct.*)
   382 
   382