src/HOL/Calculation.thy
changeset 8855 ef4848bb0696
parent 8301 d9345bad5e5c
child 9035 371f023d3dbd
equal deleted inserted replaced
8854:c2cd9e1b6142 8855:ef4848bb0696
     4 
     4 
     5 Setup transitivity rules for calculational proofs.  Note that in the
     5 Setup transitivity rules for calculational proofs.  Note that in the
     6 list below later rules have priority.
     6 list below later rules have priority.
     7 *)
     7 *)
     8 
     8 
     9 theory Calculation = Int:;
     9 theory Calculation = IntArith:;
    10 
    10 
    11 theorems [trans] = rev_mp mp;
    11 theorems [trans] = rev_mp mp;
    12 
    12 
    13 theorem [trans]: "[| s = t; P t |] ==> P s"; 		    (*  =  x  x  *)
    13 theorem [trans]: "[| s = t; P t |] ==> P s"; 		    (*  =  x  x  *)
    14   by (rule ssubst);
    14   by (rule ssubst);