src/HOL/UNITY/Comp/Alloc.thy
changeset 61853 fb7756087101
parent 60773 d09c66a0ea10
child 61954 1d43f86f48be
equal deleted inserted replaced
61852:d273c24b5776 61853:fb7756087101
   319       handle THM _ => th RS @{thm lessThanBspec}
   319       handle THM _ => th RS @{thm lessThanBspec}
   320       handle THM _ => th RS bspec
   320       handle THM _ => th RS bspec
   321       handle THM _ => th RS (@{thm guarantees_INT_right_iff} RS iffD1))
   321       handle THM _ => th RS (@{thm guarantees_INT_right_iff} RS iffD1))
   322     handle THM _ => th;
   322     handle THM _ => th;
   323 in
   323 in
   324   Scan.succeed (Thm.rule_attribute (K normalized))
   324   Scan.succeed (Thm.rule_attribute [] (K normalized))
   325 end
   325 end
   326 *}
   326 *}
   327 
   327 
   328 (*** bijectivity of sysOfAlloc [MUST BE AUTOMATED] ***)
   328 (*** bijectivity of sysOfAlloc [MUST BE AUTOMATED] ***)
   329 ML {*
   329 ML {*