src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML
changeset 60549 e168d5c48a95
parent 59058 a78612c67ec0
child 61268 abe08fb15a12
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML	Mon Jun 22 16:56:03 2015 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML	Mon Jun 22 16:56:03 2015 +0200
@@ -132,7 +132,7 @@
       (case xs of
         [] => t
       | _ =>
-        (* proof obligation: !!thesis. (!!x. A x ==> thesis) ==> thesis
+        (* proof obligation: !!thesis. (!!x1...xn. t ==> thesis) ==> thesis
            (cf. "~~/src/Pure/Isar/obtain.ML") *)
         let
           val frees = map Free xs
@@ -140,10 +140,10 @@
             Free (singleton (Variable.variant_frees ctxt frees) ("thesis", HOLogic.boolT))
           val thesis_prop = HOLogic.mk_Trueprop thesis
 
-          (* !!x1..xn. t ==> thesis (xs = [x1, .., xn]) *)
+          (* !!x1...xn. t ==> thesis *)
           val inner_prop = fold_rev Logic.all frees (Logic.mk_implies (t, thesis_prop))
         in
-          (* !!thesis. (!!x1..xn. t ==> thesis) ==> thesis *)
+          (* !!thesis. (!!x1...xn. t ==> thesis) ==> thesis *)
           Logic.all thesis (Logic.mk_implies (inner_prop, thesis_prop))
         end)