src/HOL/Library/Countable.thy
changeset 67399 eab6ce8368fa
parent 66453 cc19f7ca2ed6
child 67405 e9ab4ad7bd15
--- a/src/HOL/Library/Countable.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Library/Countable.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -180,7 +180,7 @@
         val pred_names = #names (fst induct_info)
         val induct_thms = #inducts (snd induct_info)
         val alist = pred_names ~~ induct_thms
-        val induct_thm = the (AList.lookup (op =) alist pred_name)
+        val induct_thm = the (AList.lookup (=) alist pred_name)
         val vars = rev (Term.add_vars (Thm.prop_of induct_thm) [])
         val insts = vars |> map (fn (_, T) => try (Thm.cterm_of ctxt)
           (Const (@{const_name Countable.finite_item}, T)))