src/HOL/Decision_Procs/Parametric_Ferrante_Rackoff.thy
changeset 42364 8c674b3b8e44
parent 42361 23f352990944
child 42368 3b8498ac2314
--- a/src/HOL/Decision_Procs/Parametric_Ferrante_Rackoff.thy	Sat Apr 16 16:37:21 2011 +0200
+++ b/src/HOL/Decision_Procs/Parametric_Ferrante_Rackoff.thy	Sat Apr 16 18:11:20 2011 +0200
@@ -3011,7 +3011,7 @@
  Object_Logic.full_atomize_tac i
  THEN (fn st =>
   let
-    val g = List.nth (cprems_of st, i - 1)
+    val g = nth (cprems_of st) (i - 1)
     val thy = Proof_Context.theory_of ctxt
     val fs = subtract (op aconv) (map Free (Term.add_frees (term_of g) [])) ps
     val th = frpar_oracle (T, fs,ps, (* Pattern.eta_long [] *)g)
@@ -3021,7 +3021,7 @@
  Object_Logic.full_atomize_tac i
  THEN (fn st =>
   let
-    val g = List.nth (cprems_of st, i - 1)
+    val g = nth (cprems_of st) (i - 1)
     val thy = Proof_Context.theory_of ctxt
     val fs = subtract (op aconv) (map Free (Term.add_frees (term_of g) [])) ps
     val th = frpar_oracle2 (T, fs,ps, (* Pattern.eta_long [] *)g)