src/HOL/Decision_Procs/approximation_generator.ML
author immler
Sun, 03 Nov 2019 21:46:46 -0500
changeset 71034 e0755162093f
parent 69597 ff784d5a5bfb
child 71037 f630f2e707a6
permissions -rw-r--r--
replace approximation oracle by less ad-hoc @{computation}s
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     1
(*  Title:      HOL/Decision_Procs/approximation_generator.ML
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     2
    Author:     Fabian Immler, TU Muenchen
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     3
*)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     4
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     5
signature APPROXIMATION_GENERATOR =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     6
sig
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     7
  val custom_seed: int Config.T
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     8
  val precision: int Config.T
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
     9
  val epsilon: real Config.T
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    10
  val approximation_generator:
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    11
    Proof.context ->
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    12
    (term * term list) list ->
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    13
    bool -> int list -> (bool * term list) option * Quickcheck.report option
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    14
  val setup: theory -> theory
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    15
end;
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    16
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    17
structure Approximation_Generator : APPROXIMATION_GENERATOR =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    18
struct
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    19
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    20
val custom_seed = Attrib.setup_config_int \<^binding>\<open>quickcheck_approximation_custom_seed\<close> (K ~1)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    21
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    22
val precision = Attrib.setup_config_int \<^binding>\<open>quickcheck_approximation_precision\<close> (K 30)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    23
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    24
val epsilon = Attrib.setup_config_real \<^binding>\<open>quickcheck_approximation_epsilon\<close> (K 0.0)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    25
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    26
val random_float = @{code "random_class.random::_ \<Rightarrow> _ \<Rightarrow> (float \<times> (unit \<Rightarrow> term)) \<times> _"}
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    27
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    28
fun nat_of_term t =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    29
  (HOLogic.dest_nat t handle TERM _ => snd (HOLogic.dest_number t)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    30
    handle TERM _ => raise TERM ("nat_of_term", [t]));
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    31
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    32
fun int_of_term t = snd (HOLogic.dest_number t) handle TERM _ => raise TERM ("int_of_term", [t]);
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    33
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    34
fun real_of_man_exp m e = Real.fromManExp {man = Real.fromInt m, exp = e}
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    35
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    36
fun mapprox_float (\<^term>\<open>Float\<close> $ m $ e) = real_of_man_exp (int_of_term m) (int_of_term e)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    37
  | mapprox_float t = Real.fromInt (snd (HOLogic.dest_number t))
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    38
      handle TERM _ => raise TERM ("mapprox_float", [t]);
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    39
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    40
(* TODO: define using compiled terms? *)
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    41
fun mapprox_floatarith (\<^term>\<open>Add\<close> $ a $ b) xs = mapprox_floatarith a xs + mapprox_floatarith b xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    42
  | mapprox_floatarith (\<^term>\<open>Minus\<close> $ a) xs = ~ (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    43
  | mapprox_floatarith (\<^term>\<open>Mult\<close> $ a $ b) xs = mapprox_floatarith a xs * mapprox_floatarith b xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    44
  | mapprox_floatarith (\<^term>\<open>Inverse\<close> $ a) xs = 1.0 / mapprox_floatarith a xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    45
  | mapprox_floatarith (\<^term>\<open>Cos\<close> $ a) xs = Math.cos (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    46
  | mapprox_floatarith (\<^term>\<open>Arctan\<close> $ a) xs = Math.atan (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    47
  | mapprox_floatarith (\<^term>\<open>Abs\<close> $ a) xs = abs (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    48
  | mapprox_floatarith (\<^term>\<open>Max\<close> $ a $ b) xs =
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    49
      Real.max (mapprox_floatarith a xs, mapprox_floatarith b xs)
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    50
  | mapprox_floatarith (\<^term>\<open>Min\<close> $ a $ b) xs =
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    51
      Real.min (mapprox_floatarith a xs, mapprox_floatarith b xs)
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    52
  | mapprox_floatarith \<^term>\<open>Pi\<close> _ = Math.pi
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    53
  | mapprox_floatarith (\<^term>\<open>Sqrt\<close> $ a) xs = Math.sqrt (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    54
  | mapprox_floatarith (\<^term>\<open>Exp\<close> $ a) xs = Math.exp (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    55
  | mapprox_floatarith (\<^term>\<open>Powr\<close> $ a $ b) xs =
64519
51be997d0698 op powr for quickcheck[approximation] (amending 67792e4a5486)
immler
parents: 63931
diff changeset
    56
      Math.pow (mapprox_floatarith a xs, mapprox_floatarith b xs)
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    57
  | mapprox_floatarith (\<^term>\<open>Ln\<close> $ a) xs = Math.ln (mapprox_floatarith a xs)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    58
  | mapprox_floatarith (\<^term>\<open>Power\<close> $ a $ n) xs =
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    59
      Math.pow (mapprox_floatarith a xs, Real.fromInt (nat_of_term n))
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    60
  | mapprox_floatarith (\<^term>\<open>Floor\<close> $ a) xs = Real.fromInt (floor (mapprox_floatarith a xs))
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    61
  | mapprox_floatarith (\<^term>\<open>Var\<close> $ n) xs = nth xs (nat_of_term n)
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    62
  | mapprox_floatarith (\<^term>\<open>Num\<close> $ m) _ = mapprox_float m
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    63
  | mapprox_floatarith t _ = raise TERM ("mapprox_floatarith", [t])
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    64
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    65
fun mapprox_atLeastAtMost eps x a b xs =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    66
    let
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    67
      val x' = mapprox_floatarith x xs
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    68
    in
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    69
      mapprox_floatarith a xs + eps <= x' andalso x' + eps <= mapprox_floatarith b xs
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    70
    end
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    71
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    72
fun mapprox_form eps (\<^term>\<open>Bound\<close> $ x $ a $ b $ f) xs =
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    73
    (not (mapprox_atLeastAtMost eps x a b xs)) orelse mapprox_form eps f xs
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    74
| mapprox_form eps (\<^term>\<open>Assign\<close> $ x $ a $ f) xs =
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    75
    (Real.!= (mapprox_floatarith x xs, mapprox_floatarith a xs)) orelse mapprox_form eps f xs
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    76
| mapprox_form eps (\<^term>\<open>Less\<close> $ a $ b) xs = mapprox_floatarith a xs + eps < mapprox_floatarith b xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    77
| mapprox_form eps (\<^term>\<open>LessEqual\<close> $ a $ b) xs = mapprox_floatarith a xs + eps <= mapprox_floatarith b xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    78
| mapprox_form eps (\<^term>\<open>AtLeastAtMost\<close> $ x $ a $ b) xs = mapprox_atLeastAtMost eps x a b xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    79
| mapprox_form eps (\<^term>\<open>Conj\<close> $ f $ g) xs = mapprox_form eps f xs andalso mapprox_form eps g xs
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    80
| mapprox_form eps (\<^term>\<open>Disj\<close> $ f $ g) xs = mapprox_form eps f xs orelse mapprox_form eps g xs
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    81
| mapprox_form _ t _ = raise TERM ("mapprox_form", [t])
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    82
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    83
fun dest_interpret_form (\<^const>\<open>interpret_form\<close> $ b $ xs) = (b, xs)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    84
  | dest_interpret_form t = raise TERM ("dest_interpret_form", [t])
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    85
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    86
fun optionT t = Type (\<^type_name>\<open>option\<close>, [t])
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    87
fun mk_Some t = Const (\<^const_name>\<open>Some\<close>, t --> optionT t)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    88
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    89
fun random_float_list size xs seed =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    90
  fold (K (apsnd (random_float size) #-> (fn c => apfst (fn b => b::c)))) xs ([],seed)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    91
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    92
fun real_of_Float (@{code Float} (m, e)) =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    93
    real_of_man_exp (@{code integer_of_int} m) (@{code integer_of_int} e)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
    94
71034
e0755162093f replace approximation oracle by less ad-hoc @{computation}s
immler
parents: 69597
diff changeset
    95
fun term_of_int i = (HOLogic.mk_number @{typ int} (@{code integer_of_int} i))
e0755162093f replace approximation oracle by less ad-hoc @{computation}s
immler
parents: 69597
diff changeset
    96
e0755162093f replace approximation oracle by less ad-hoc @{computation}s
immler
parents: 69597
diff changeset
    97
fun term_of_Float (@{code Float} (m, e)) = @{term Float} $ term_of_int m $ term_of_int e
e0755162093f replace approximation oracle by less ad-hoc @{computation}s
immler
parents: 69597
diff changeset
    98
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
    99
fun is_True \<^term>\<open>True\<close> = true
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   100
  | is_True _ = false
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   101
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   102
val postproc_form_eqs =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   103
  @{lemma
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   104
    "real_of_float (Float 0 a) = 0"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   105
    "real_of_float (Float (numeral m) 0) = numeral m"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   106
    "real_of_float (Float 1 0) = 1"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   107
    "real_of_float (Float (- 1) 0) = - 1"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   108
    "real_of_float (Float 1 (numeral e)) = 2 ^ numeral e"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   109
    "real_of_float (Float 1 (- numeral e)) = 1 / 2 ^ numeral e"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   110
    "real_of_float (Float a 1) = a * 2"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   111
    "real_of_float (Float a (-1)) = a / 2"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   112
    "real_of_float (Float (- a) b) = - real_of_float (Float a b)"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   113
    "real_of_float (Float (numeral m) (numeral e)) = numeral m * 2 ^ (numeral e)"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 59850
diff changeset
   114
    "real_of_float (Float (numeral m) (- numeral e)) = numeral m / 2 ^ (numeral e)"
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   115
    "- (c * d::real) = -c * d"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   116
    "- (c / d::real) = -c / d"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   117
    "- (0::real) = 0"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   118
    "int_of_integer (numeral k) = numeral k"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   119
    "int_of_integer (- numeral k) = - numeral k"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   120
    "int_of_integer 0 = 0"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   121
    "int_of_integer 1 = 1"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   122
    "int_of_integer (- 1) = - 1"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   123
    by auto
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   124
  }
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   125
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   126
fun rewrite_with ctxt thms = Simplifier.rewrite (put_simpset HOL_basic_ss ctxt addsimps thms)
59629
0d77c51b5040 clarified context;
wenzelm
parents: 59621
diff changeset
   127
fun conv_term ctxt conv r = Thm.cterm_of ctxt r |> conv |> Thm.prop_of |> Logic.dest_equals |> snd
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   128
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   129
fun approx_random ctxt prec eps frees e xs genuine_only size seed =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   130
  let
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   131
    val (rs, seed') = random_float_list size xs seed
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   132
    fun mk_approx_form e ts =
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   133
      \<^const>\<open>approx_form\<close> $
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   134
        HOLogic.mk_number \<^typ>\<open>nat\<close> prec $
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   135
        e $
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   136
        (HOLogic.mk_list \<^typ>\<open>(float * float) option\<close>
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   137
          (map (fn t => mk_Some \<^typ>\<open>float * float\<close> $ HOLogic.mk_prod (t, t)) ts)) $
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   138
        \<^term>\<open>[] :: nat list\<close>
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   139
  in
63931
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   140
    (if
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   141
      mapprox_form eps e (map (real_of_Float o fst) rs)
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   142
      handle
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   143
        General.Overflow => false
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   144
      | General.Domain => false
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   145
      | General.Div => false
f17a1c60ac39 approximation: preprocessing for nat/int expressions
immler
parents: 63929
diff changeset
   146
      | IEEEReal.Unordered => false
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   147
    then
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   148
      let
71034
e0755162093f replace approximation oracle by less ad-hoc @{computation}s
immler
parents: 69597
diff changeset
   149
        val ts = map (fn x => term_of_Float (fst x)) rs
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   150
        val ts' = map
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   151
          (AList.lookup op = (map dest_Free xs ~~ ts)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   152
            #> the_default Term.dummy
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   153
            #> curry op $ \<^term>\<open>real_of_float::float\<Rightarrow>_\<close>
59629
0d77c51b5040 clarified context;
wenzelm
parents: 59621
diff changeset
   154
            #> conv_term ctxt (rewrite_with ctxt postproc_form_eqs))
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   155
          frees
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   156
      in
59850
f339ff48a6ee exposed approximation in ML
eberlm
parents: 59629
diff changeset
   157
        if Approximation.approximate ctxt (mk_approx_form e ts) |> is_True
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   158
        then SOME (true, ts')
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   159
        else (if genuine_only then NONE else SOME (false, ts'))
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   160
      end
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   161
    else NONE, seed')
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   162
  end
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   163
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   164
val preproc_form_eqs =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   165
  @{lemma
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   166
    "(a::real) \<in> {b .. c} \<longleftrightarrow> b \<le> a \<and> a \<le> c"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   167
    "a = b \<longleftrightarrow> a \<le> b \<and> b \<le> a"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   168
    "(p \<longrightarrow> q) \<longleftrightarrow> \<not>p \<or> q"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   169
    "(p \<longleftrightarrow> q) \<longleftrightarrow> (p \<longrightarrow> q) \<and> (q \<longrightarrow> p)"
59629
0d77c51b5040 clarified context;
wenzelm
parents: 59621
diff changeset
   170
    by auto}
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   171
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   172
fun reify_goal ctxt t =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   173
  HOLogic.mk_not t
59629
0d77c51b5040 clarified context;
wenzelm
parents: 59621
diff changeset
   174
    |> conv_term ctxt (rewrite_with ctxt preproc_form_eqs)
63929
b673e7221b16 approximation: rewrite for reduction to base expressions
immler
parents: 61609
diff changeset
   175
    |> Approximation.reify_form ctxt
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   176
    |> dest_interpret_form
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   177
    ||> HOLogic.dest_list
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   178
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   179
fun approximation_generator_raw ctxt t =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   180
  let
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   181
    val iterations = Config.get ctxt Quickcheck.iterations
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   182
    val prec = Config.get ctxt precision
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   183
    val eps = Config.get ctxt epsilon
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   184
    val cs = Config.get ctxt custom_seed
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   185
    val seed = (Code_Numeral.natural_of_integer (cs + 1), Code_Numeral.natural_of_integer 1)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   186
    val run = if cs < 0
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   187
      then (fn f => fn seed => (Random_Engine.run f, seed))
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   188
      else (fn f => fn seed => f seed)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   189
    val frees = Term.add_frees t []
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   190
    val (e, xs) = reify_goal ctxt t
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   191
    fun single_tester b s =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   192
      approx_random ctxt prec eps frees e xs b s |> run
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   193
    fun iterate _ _ 0 _ = NONE
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   194
      | iterate genuine_only size j seed =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   195
        case single_tester genuine_only size seed of
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   196
          (NONE, seed') => iterate genuine_only size (j - 1) seed'
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   197
        | (SOME q, _) => SOME q
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   198
  in
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   199
    fn genuine_only => fn size => (iterate genuine_only size iterations seed, NONE)
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   200
  end
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   201
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   202
fun approximation_generator ctxt [(t, _)] =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   203
  (fn genuine_only =>
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   204
    fn [_, size] =>
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   205
      approximation_generator_raw ctxt t genuine_only
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   206
        (Code_Numeral.natural_of_integer size))
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   207
  | approximation_generator _ _ =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   208
      error "Quickcheck-approximation does not support type variables (or finite instantiations)"
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   209
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   210
val test_goals =
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   211
  Quickcheck_Common.generator_test_goal_terms
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   212
    ("approximation", (fn _ => fn _ => false, approximation_generator))
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   213
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 64519
diff changeset
   214
val active = Attrib.setup_config_bool \<^binding>\<open>quickcheck_approximation_active\<close> (K false)
58988
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   215
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   216
val setup = Context.theory_map (Quickcheck.add_tester ("approximation", (active, test_goals)))
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   217
6ebf918128b9 added quickcheck[approximation]
immler
parents:
diff changeset
   218
end