src/HOL/Tools/numeral.ML
changeset 54489 03ff4d1e6784
parent 52435 6646bb548c6b
child 55147 bce3dbc11f95
--- a/src/HOL/Tools/numeral.ML	Tue Nov 19 01:30:14 2013 +0100
+++ b/src/HOL/Tools/numeral.ML	Tue Nov 19 10:05:53 2013 +0100
@@ -45,8 +45,8 @@
 val numeral = @{cpat "numeral"};
 val numeralT = Thm.ctyp_of @{theory} (Term.range_type (Thm.typ_of (Thm.ctyp_of_term numeral)));
 
-val neg_numeral = @{cpat "neg_numeral"};
-val neg_numeralT = Thm.ctyp_of @{theory} (Term.range_type (Thm.typ_of (Thm.ctyp_of_term neg_numeral)));
+val uminus = @{cpat "uminus"};
+val uminusT = Thm.ctyp_of @{theory} (Term.range_type (Thm.typ_of (Thm.ctyp_of_term uminus)));
 
 fun instT T V = Thm.instantiate_cterm ([(V, T)], []);
 
@@ -56,7 +56,7 @@
   | mk_cnumber T 1 = instT T oneT one
   | mk_cnumber T i =
     if i > 0 then Thm.apply (instT T numeralT numeral) (mk_cnumeral i)
-    else Thm.apply (instT T neg_numeralT neg_numeral) (mk_cnumeral (~i));
+    else Thm.apply (instT T uminusT uminus) (Thm.apply (instT T numeralT numeral) (mk_cnumeral (~i)));
 
 end;