src/HOL/Tools/SMT/z3_proof_tools.ML
changeset 38795 848be46708dc
parent 38786 e46e7a9cb622
child 38864 4abe644fcea5
equal deleted inserted replaced
38794:2d638e963357 38795:848be46708dc
   194         @{term Trueprop} $ _ => abstr1 cvs ct
   194         @{term Trueprop} $ _ => abstr1 cvs ct
   195       | @{term "op ==>"} $ _ $ _ => abstr2 cvs ct
   195       | @{term "op ==>"} $ _ $ _ => abstr2 cvs ct
   196       | @{term True} => pair ct
   196       | @{term True} => pair ct
   197       | @{term False} => pair ct
   197       | @{term False} => pair ct
   198       | @{term Not} $ _ => abstr1 cvs ct
   198       | @{term Not} $ _ => abstr1 cvs ct
   199       | @{term "op &"} $ _ $ _ => abstr2 cvs ct
   199       | @{term HOL.conj} $ _ $ _ => abstr2 cvs ct
   200       | @{term "op |"} $ _ $ _ => abstr2 cvs ct
   200       | @{term HOL.disj} $ _ $ _ => abstr2 cvs ct
   201       | @{term HOL.implies} $ _ $ _ => abstr2 cvs ct
   201       | @{term HOL.implies} $ _ $ _ => abstr2 cvs ct
   202       | Const (@{const_name "op ="}, _) $ _ $ _ => abstr2 cvs ct
   202       | Const (@{const_name "op ="}, _) $ _ $ _ => abstr2 cvs ct
   203       | Const (@{const_name distinct}, _) $ _ =>
   203       | Const (@{const_name distinct}, _) $ _ =>
   204           if ext_logic then abs_arg (abs_list abstr fresh_abstraction) cvs ct
   204           if ext_logic then abs_arg (abs_list abstr fresh_abstraction) cvs ct
   205           else fresh_abstraction cvs ct
   205           else fresh_abstraction cvs ct