eliminated old numerals;
authorwenzelm
Tue, 23 Oct 2001 22:52:31 +0200
changeset 11908 82f68fd05094
parent 11907 f2a5481c7998
child 11909 92e442b783db
eliminated old numerals;
src/HOL/MicroJava/J/Example.thy
src/HOL/MicroJava/J/Value.thy
src/HOL/ex/AVL.thy
--- a/src/HOL/MicroJava/J/Example.thy	Tue Oct 23 22:51:30 2001 +0200
+++ b/src/HOL/MicroJava/J/Example.thy	Tue Oct 23 22:52:31 2001 +0200
@@ -100,7 +100,7 @@
 			     [(vee, PrimT Boolean)], 
 			     [((foo,[Class Base]),Class Base,foo_Base)]))"
   foo_Ext_def:"foo_Ext == ([x],[],Expr( {Ext}Cast Ext
-				       (LAcc x)..vee:=Lit (Intg Numeral1)),
+				       (LAcc x)..vee:=Lit (Intg 1)),
 				   Lit Null)"
   ExtC_def: "ExtC  == (Ext,  (Base  , 
 			     [(vee, PrimT Integer)], 
@@ -127,7 +127,7 @@
   "NP"   == "NullPointer"
   "tprg" == "[ObjectC, BaseC, ExtC]"
   "obj1"    <= "(Ext, empty((vee, Base)\<mapsto>Bool False)
-			   ((vee, Ext )\<mapsto>Intg Numeral0))"
+			   ((vee, Ext )\<mapsto>Intg 0))"
   "s0" == " Norm    (empty, empty)"
   "s1" == " Norm    (empty(a\<mapsto>obj1),empty(e\<mapsto>Addr a))"
   "s2" == " Norm    (empty(a\<mapsto>obj1),empty(x\<mapsto>Null)(This\<mapsto>Addr a))"
--- a/src/HOL/MicroJava/J/Value.thy	Tue Oct 23 22:51:30 2001 +0200
+++ b/src/HOL/MicroJava/J/Value.thy	Tue Oct 23 22:52:31 2001 +0200
@@ -40,7 +40,7 @@
 primrec
   "defpval Void    = Unit"
   "defpval Boolean = Bool False"
-  "defpval Integer = Intg (Numeral0)"
+  "defpval Integer = Intg 0"
 
 primrec
   "default_val (PrimT pt) = defpval pt"
--- a/src/HOL/ex/AVL.thy	Tue Oct 23 22:51:30 2001 +0200
+++ b/src/HOL/ex/AVL.thy	Tue Oct 23 22:52:31 2001 +0200
@@ -6,7 +6,7 @@
 AVL trees: at the moment only insertion.
 This version works exclusively with nat.
 Balance check could be simplified by working with int:
-"isbal (MKT n l r) = (abs(int(height l) - int(height r)) <= Numeral1 &
+"isbal (MKT n l r) = (abs(int(height l) - int(height r)) <= 1 &
                       isbal l & isbal r)"
 *)