diff -r eb2caacf3ba4 -r a8e96847523c src/HOL/Import/HOL_Light_Maps.thy --- a/src/HOL/Import/HOL_Light_Maps.thy Wed Feb 12 08:35:56 2014 +0100 +++ b/src/HOL/Import/HOL_Light_Maps.thy Wed Feb 12 08:35:56 2014 +0100 @@ -230,7 +230,7 @@ lemma list_RECURSION: "\nil' cons'. \fn\'A list \ 'Z. fn [] = nil' \ (\(a0\'A) a1\'A list. fn (a0 # a1) = cons' a0 a1 (fn a1))" - by (intro allI, rule_tac x="list_rec nil' cons'" in exI) auto + by (intro allI, rule_tac x="rec_list nil' cons'" in exI) auto lemma HD[import_const HD : List.hd]: "hd ((h\'A) # t) = h"