proper p' instead of p (amending 52c7c42e7e27);
authorwenzelm
Fri, 15 Oct 2021 21:10:54 +0200
changeset 74527 52eadb60499f
parent 74526 bbfed17243af
child 74528 ce2c7037e509
proper p' instead of p (amending 52c7c42e7e27);
src/HOL/Decision_Procs/Cooper.thy
--- a/src/HOL/Decision_Procs/Cooper.thy	Fri Oct 15 20:54:13 2021 +0200
+++ b/src/HOL/Decision_Procs/Cooper.thy	Fri Oct 15 21:10:54 2021 +0200
@@ -2427,16 +2427,16 @@
       @{code Imp} (fm_of_term ps vs t1, fm_of_term ps vs t2)
   | fm_of_term ps vs \<^Const_>\<open>HOL.Not for t'\<close> =
       @{code Not} (fm_of_term ps vs t')
-  | fm_of_term ps vs \<^Const_>\<open>Ex _ for \<open>t as Abs (_, _, p)\<close>\<close> =
+  | fm_of_term ps vs \<^Const_>\<open>Ex _ for \<open>t as Abs _\<close>\<close> =
       let
         val (x', p') = Term.dest_abs_global t;
         val vs' = (Free x', 0) :: map (fn (v, n) => (v, n + 1)) vs;
-      in @{code E} (fm_of_term ps vs' p) end
-  | fm_of_term ps vs \<^Const_>\<open>All _ for \<open>t as Abs (_, _, p)\<close>\<close> =
+      in @{code E} (fm_of_term ps vs' p') end
+  | fm_of_term ps vs \<^Const_>\<open>All _ for \<open>t as Abs _\<close>\<close> =
       let
         val (x', p') = Term.dest_abs_global t;
         val vs' = (Free x', 0) :: map (fn (v, n) => (v, n + 1)) vs;
-      in @{code A} (fm_of_term ps vs' p) end
+      in @{code A} (fm_of_term ps vs' p') end
   | fm_of_term ps vs t = error ("fm_of_term : unknown term " ^ Syntax.string_of_term \<^context> t);
 
 fun term_of_num vs (@{code C} i) = HOLogic.mk_number HOLogic.intT (@{code integer_of_int} i)