code generator: wfrec combinator is now implemented by ML function wf_rec.
authorberghofe
Fri, 19 Apr 2002 14:51:33 +0200
changeset 13093 ab0335307905
parent 13092 eae72c47d07f
child 13094 643fce75f6cd
code generator: wfrec combinator is now implemented by ML function wf_rec.
src/HOL/Main.thy
--- a/src/HOL/Main.thy	Fri Apr 19 14:47:10 2002 +0200
+++ b/src/HOL/Main.thy	Fri Apr 19 14:51:33 2002 +0200
@@ -116,6 +116,10 @@
   "Nil"     ("[]")
   "Cons"    ("(_ ::/ _)")
 
+  "wfrec"   ("wf'_rec?")
+
+ML {* fun wf_rec f x = f (wf_rec f) x; *}
+
 lemma [code]: "((n::nat) < 0) = False" by simp
 declare less_Suc_eq [code]