use aconv to compare terms (for cleanliness)
authorblanchet
Mon, 03 Mar 2014 12:48:19 +0100
changeset 55853 e776a4b813d1
parent 55852 48ced935c0e5
child 55854 ee270328a781
use aconv to compare terms (for cleanliness)
src/HOL/Tools/BNF/bnf_comp.ML
--- a/src/HOL/Tools/BNF/bnf_comp.ML	Mon Mar 03 12:48:19 2014 +0100
+++ b/src/HOL/Tools/BNF/bnf_comp.ML	Mon Mar 03 12:48:19 2014 +0100
@@ -97,7 +97,7 @@
 
 fun is_sum_prod_natLeq (Const (@{const_name csum}, _) $ t $ u) = forall is_sum_prod_natLeq [t, u]
   | is_sum_prod_natLeq (Const (@{const_name cprod}, _) $ t $ u) = forall is_sum_prod_natLeq [t, u]
-  | is_sum_prod_natLeq t = (t = @{term natLeq});
+  | is_sum_prod_natLeq t = t aconv @{term natLeq};
 
 fun clean_compose_bnf const_policy qualify b outer inners (unfold_set, lthy) =
   let