changeset 58957 | c9e744ea8a38 |
parent 58956 | a816aa3ff391 |
child 58958 | 114255dce178 |
--- a/src/HOL/HOL.thy Sun Nov 09 14:08:00 2014 +0100 +++ b/src/HOL/HOL.thy Sun Nov 09 17:04:14 2014 +0100 @@ -1463,7 +1463,7 @@ val equal_def = @{thm induct_equal_def} fun dest_def (Const (@{const_name induct_equal}, _) $ t $ u) = SOME (t, u) | dest_def _ = NONE - val trivial_tac = match_tac @{thms induct_trueI} + fun trivial_tac ctxt = match_tac ctxt @{thms induct_trueI} ) *}