Adapted to new name mangling function in code generator.
--- a/src/HOL/Lambda/WeakNorm.thy Tue Jun 01 14:59:54 2004 +0200
+++ b/src/HOL/Lambda/WeakNorm.thy Tue Jun 01 15:00:26 2004 +0200
@@ -535,10 +535,10 @@
*}
ML {*
-fun nat_of_int 0 = id0
+fun nat_of_int 0 = id_0
| nat_of_int n = Suc (nat_of_int (n-1));
-fun int_of_nat id0 = 0
+fun int_of_nat id_0 = 0
| int_of_nat (Suc n) = 1 + int_of_nat n;
fun dBtype_of_typ (Type ("fun", [T, U])) =
@@ -576,7 +576,7 @@
let val dBT = dBtype_of_typ T
in rtypingT_Abs (e, dBT, dB_of_term t,
dBtype_of_typ (fastype_of1 (T :: Ts, t)),
- typing_of_term (T :: Ts) (shift e id0 dBT) t)
+ typing_of_term (T :: Ts) (shift e id_0 dBT) t)
end
| typing_of_term _ _ _ = error "typing_of_term: bad term";