# HG changeset patch # User haftmann # Date 1158672123 -7200 # Node ID 3950e65f48f89c9ccfff6d49c582077ced460891 # Parent db6bedfba49828a834b21b093de745b0d1997901 (void) diff -r db6bedfba498 -r 3950e65f48f8 src/HOL/Integ/Numeral.thy --- a/src/HOL/Integ/Numeral.thy Tue Sep 19 15:21:58 2006 +0200 +++ b/src/HOL/Integ/Numeral.thy Tue Sep 19 15:22:03 2006 +0200 @@ -441,6 +441,7 @@ by (simp add: neg_def number_of_eq numeral_simps double_less_0_iff Ints_odd_less_0 Ints_def split: bit.split) + text {* Less-Than or Equals *} text {* Reduces @{term "a\b"} to @{term "~ (b Univ) * (Univ list) * int * (unit -> nterm); fun to_term (Constr(name, args)) = apps (C name) (map to_term args) - | to_term (Var (name, args)) = apps (V name) (map to_term args) - | to_term (BVar (name, args)) = apps (B name) (map to_term args) - | to_term (Fun(_,args,_,name_thunk)) = apps (name_thunk ()) (map to_term args); + | to_term (Var (name, args)) = apps (V name) (map to_term args) + | to_term (BVar (name, args)) = apps (B name) (map to_term args) + | to_term (Fun(_,args,_,name_thunk)) = apps (name_thunk ()) (map to_term args); (* A typical operation, why functions might be good for, is