abstraction over functions is no default any more.
authorchaieb
Wed, 26 May 2004 19:06:09 +0200
changeset 14811 9144ec118703
parent 14810 4b4b97d29370
child 14812 4b2c006d0534
abstraction over functions is no default any more.
src/HOL/Integ/presburger.ML
src/HOL/Tools/Presburger/presburger.ML
--- a/src/HOL/Integ/presburger.ML	Wed May 26 18:52:18 2004 +0200
+++ b/src/HOL/Integ/presburger.ML	Wed May 26 19:06:09 2004 +0200
@@ -6,7 +6,7 @@
 Tactic for solving arithmetical Goals in Presburger Arithmetic
 *)
 
-(* This version of presburger deals with occurences of functional symbols in the subgoal and abstract over them to try to prove the more general formula. It then resolves with the subgoal. To disable this feature call the procedure with the parameter no_abs
+(* This version of presburger deals with occurences of functional symbols in the subgoal and abstract over them to try to prove the more general formula. It then resolves with the subgoal. To enable this feature call the procedure with the parameter abs
 *)
 
 signature PRESBURGER = 
@@ -279,11 +279,11 @@
 fun presburger_args meth =
  let val parse_flag = 
          Args.$$$ "no_quantify" >> K (apfst (K false))
-      || Args.$$$ "no_abs" >> K (apsnd (K false));
+      || Args.$$$ "abs" >> K (apsnd (K true));
  in
    Method.simple_args 
   (Scan.optional (Args.$$$ "(" |-- Args.list1 parse_flag --| Args.$$$ ")") [] >>
-    curry (foldl op |>) (true, true))
+    curry (foldl op |>) (true, false))
     (fn (q,a) => fn _ => meth q a 1)
   end;
 
@@ -296,7 +296,7 @@
      "decision procedure for Presburger arithmetic"),
    ArithTheoryData.map (fn {splits, inj_consts, discrete, presburger} =>
      {splits = splits, inj_consts = inj_consts, discrete = discrete,
-      presburger = Some (presburger_tac true true)})];
+      presburger = Some (presburger_tac true false)})];
 
 end;
 
--- a/src/HOL/Tools/Presburger/presburger.ML	Wed May 26 18:52:18 2004 +0200
+++ b/src/HOL/Tools/Presburger/presburger.ML	Wed May 26 19:06:09 2004 +0200
@@ -6,7 +6,7 @@
 Tactic for solving arithmetical Goals in Presburger Arithmetic
 *)
 
-(* This version of presburger deals with occurences of functional symbols in the subgoal and abstract over them to try to prove the more general formula. It then resolves with the subgoal. To disable this feature call the procedure with the parameter no_abs
+(* This version of presburger deals with occurences of functional symbols in the subgoal and abstract over them to try to prove the more general formula. It then resolves with the subgoal. To enable this feature call the procedure with the parameter abs
 *)
 
 signature PRESBURGER = 
@@ -279,11 +279,11 @@
 fun presburger_args meth =
  let val parse_flag = 
          Args.$$$ "no_quantify" >> K (apfst (K false))
-      || Args.$$$ "no_abs" >> K (apsnd (K false));
+      || Args.$$$ "abs" >> K (apsnd (K true));
  in
    Method.simple_args 
   (Scan.optional (Args.$$$ "(" |-- Args.list1 parse_flag --| Args.$$$ ")") [] >>
-    curry (foldl op |>) (true, true))
+    curry (foldl op |>) (true, false))
     (fn (q,a) => fn _ => meth q a 1)
   end;
 
@@ -296,7 +296,7 @@
      "decision procedure for Presburger arithmetic"),
    ArithTheoryData.map (fn {splits, inj_consts, discrete, presburger} =>
      {splits = splits, inj_consts = inj_consts, discrete = discrete,
-      presburger = Some (presburger_tac true true)})];
+      presburger = Some (presburger_tac true false)})];
 
 end;