src/HOL/Tools/Function/termination.ML
changeset 32135 f645b51e8e54
parent 31971 8c1b845ed105
child 32149 ef59550a55d3
--- a/src/HOL/Tools/Function/termination.ML	Wed Jul 22 14:20:32 2009 +0200
+++ b/src/HOL/Tools/Function/termination.ML	Wed Jul 22 14:20:32 2009 +0200
@@ -145,7 +145,7 @@
 
 fun mk_sum_skel rel =
   let
-    val cs = FundefLib.dest_binop_list @{const_name Un} rel
+    val cs = FundefLib.dest_binop_list @{const_name union} rel
     fun collect_pats (Const ("Collect", _) $ Abs (_, _, c)) =
       let
         val (Const ("op &", _) $ (Const ("op =", _) $ _ $ (Const ("Pair", _) $ r $ l)) $ Gam)
@@ -233,7 +233,7 @@
 fun CALLS tac i st =
   if Thm.no_prems st then all_tac st
   else case Thm.term_of (Thm.cprem_of st i) of
-    (_ $ (_ $ rel)) => tac (FundefLib.dest_binop_list @{const_name Un} rel, i) st
+    (_ $ (_ $ rel)) => tac (FundefLib.dest_binop_list @{const_name union} rel, i) st
   |_ => no_tac st
 
 type ttac = (data -> int -> tactic) -> (data -> int -> tactic) -> data -> int -> tactic
@@ -293,7 +293,7 @@
           if null ineqs then
               Const (@{const_name Set.empty}, fastype_of rel)
           else
-              foldr1 (HOLogic.mk_binop @{const_name Un}) (map mk_compr ineqs)
+              foldr1 (HOLogic.mk_binop @{const_name union}) (map mk_compr ineqs)
 
       fun solve_membership_tac i =
           (EVERY' (replicate (i - 2) (rtac @{thm UnI2}))  (* pick the right component of the union *)