| changeset 58421 | 37cbbd8eb460 |
| parent 58410 | 6d46ad54a2ab |
| child 58512 | dc4d76dfa8f0 |
--- a/src/HOL/Num.thy Mon Sep 22 17:07:18 2014 +0200 +++ b/src/HOL/Num.thy Mon Sep 22 21:28:57 2014 +0200 @@ -287,7 +287,7 @@ fun numeral_tr [(c as Const (@{syntax_const "_constrain"}, _)) $ t $ u] = c $ numeral_tr [t] $ u | numeral_tr [Const (num, _)] = - (Numeral.mk_number_syntax o #value o Lexicon.read_xnum) num + (Numeral.mk_number_syntax o #value o Lexicon.read_num) num | numeral_tr ts = raise TERM ("numeral_tr", ts); in [(@{syntax_const "_Numeral"}, K numeral_tr)] end *}