fixed recdef, broken by my previous commit
authorkrauss
Sat, 26 Apr 2008 08:49:31 +0200
changeset 26750 b53db47a43b4
parent 26749 397a1aeede7d
child 26751 2b97ea3130c2
fixed recdef, broken by my previous commit
src/HOL/Tools/TFL/rules.ML
src/HOL/Tools/TFL/usyntax.ML
--- a/src/HOL/Tools/TFL/rules.ML	Fri Apr 25 16:28:06 2008 +0200
+++ b/src/HOL/Tools/TFL/rules.ML	Sat Apr 26 08:49:31 2008 +0200
@@ -458,7 +458,7 @@
 fun is_cong thm =
   case (Thm.prop_of thm)
      of (Const("==>",_)$(Const("Trueprop",_)$ _) $
-         (Const("==",_) $ (Const ("Wellfounded_Recursion.cut",_) $ f $ R $ a $ x) $ _)) => false
+         (Const("==",_) $ (Const (@{const_name "Wellfounded.cut"},_) $ f $ R $ a $ x) $ _)) => false
       | _ => true;
 
 
@@ -661,7 +661,7 @@
   end;
 
 fun restricted t = isSome (S.find_term
-                            (fn (Const("Wellfounded_Recursion.cut",_)) =>true | _ => false)
+                            (fn (Const(@{const_name "Wellfounded.cut"},_)) =>true | _ => false)
                             t)
 
 fun CONTEXT_REWRITE_RULE (func, G, cut_lemma, congs) th =
--- a/src/HOL/Tools/TFL/usyntax.ML	Fri Apr 25 16:28:06 2008 +0200
+++ b/src/HOL/Tools/TFL/usyntax.ML	Sat Apr 26 08:49:31 2008 +0200
@@ -400,7 +400,7 @@
         end handle Bind => raise USYN_ERR "dest_relation" "unexpected term structure"
    else raise USYN_ERR "dest_relation" "not a boolean term";
 
-fun is_WFR (Const("Wellfounded_Recursion.wf",_)$_) = true
+fun is_WFR (Const(@{const_name "Wellfounded.wf"},_)$_) = true
   | is_WFR _                 = false;
 
 fun ARB ty = mk_select{Bvar=Free("v",ty),