Nominal/nominal_function.ML
author Christian Urban <christian dot urban at kcl dot ac dot uk>
Mon, 19 May 2014 11:19:48 +0100
changeset 3234 08c3ef07cef7
parent 3233 9ae285ce814e
child 3235 5ebd327ffb96
permissions -rw-r--r--
changes from upstream
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     1
(*  Nominal Mutual Functions
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     2
    Author:  Christian Urban
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     3
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     4
    heavily based on the code of Alexander Krauss
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     5
    (code forked on 14 January 2011)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     6
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     7
Main entry points to the nominal function package.
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     8
*)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     9
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    10
signature NOMINAL_FUNCTION =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    11
sig
2973
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
    12
  include NOMINAL_FUNCTION_DATA
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    13
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    14
  val add_nominal_function: (binding * typ option * mixfix) list ->
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
    15
    (Attrib.binding * term) list ->  Nominal_Function_Common.nominal_function_config ->
2973
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
    16
    (Proof.context -> tactic) -> local_theory -> nominal_info * local_theory
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    17
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    18
  val add_nominal_function_cmd: (binding * string option * mixfix) list ->
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
    19
    (Attrib.binding * string) list ->  Nominal_Function_Common.nominal_function_config ->
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
    20
    (Proof.context -> tactic) -> bool -> local_theory -> nominal_info * local_theory
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    21
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    22
  val nominal_function: (binding * typ option * mixfix) list ->
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
    23
    (Attrib.binding * term) list ->  Nominal_Function_Common.nominal_function_config ->
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    24
    local_theory -> Proof.state
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    25
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    26
  val nominal_function_cmd: (binding * string option * mixfix) list ->
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
    27
    (Attrib.binding * string) list ->  Nominal_Function_Common.nominal_function_config ->
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
    28
    bool -> local_theory -> Proof.state
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    29
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    30
  val setup : theory -> theory
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    31
  val get_congs : Proof.context -> thm list
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    32
2973
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
    33
  val get_info : Proof.context -> term -> nominal_info
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    34
end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    35
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    36
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    37
structure Nominal_Function : NOMINAL_FUNCTION =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    38
struct
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    39
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    40
open Function_Lib
2821
c7d4bd9e89e0 fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents: 2819
diff changeset
    41
open Function_Common
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
    42
open Nominal_Function_Common
2752
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    43
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    44
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    45
(* Check for all sorts of errors in the input - nominal needs a different checking function *)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    46
fun nominal_check_defs ctxt fixes eqs =
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    47
  let
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    48
    val fnames = map (fst o fst) fixes
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    49
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    50
    fun check geq =
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    51
      let
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    52
        fun input_error msg = error (cat_lines [msg, Syntax.string_of_term ctxt geq])
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    53
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    54
        fun check_head fname =
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    55
          member (op =) fnames fname orelse
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    56
          input_error ("Illegal equation head. Expected " ^ commas_quote fnames)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    57
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    58
        val (fname, qs, gs, args, rhs) = split_def ctxt check_head geq
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    59
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    60
        val _ = length args > 0 orelse input_error "Function has no arguments:"
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    61
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    62
        fun add_bvs t is = add_loose_bnos (t, 0, is)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    63
        val rvs = (subtract (op =) (fold add_bvs args []) (add_bvs rhs []))
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    64
                    |> map (fst o nth (rev qs))
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    65
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    66
        val _ = forall (not o Term.exists_subterm
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    67
          (fn Free (n, _) => member (op =) fnames n | _ => false)) (gs @ args)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    68
          orelse input_error "Defined function may not occur in premises or arguments"
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    69
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    70
        val freeargs = map (fn t => subst_bounds (rev (map Free qs), t)) args
2860
25a7f421a3ba added a test that every function must be of pt-sort
Christian Urban <urbanc@in.tum.de>
parents: 2821
diff changeset
    71
        val funvars = filter (fn q => 
25a7f421a3ba added a test that every function must be of pt-sort
Christian Urban <urbanc@in.tum.de>
parents: 2821
diff changeset
    72
          exists (exists_subterm (fn (Free q') $ _ => q = q' | _ => false)) freeargs) qs
2752
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    73
        val _ = null funvars orelse (warning (cat_lines
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    74
          ["Bound variable" ^ plural " " "s " funvars ^
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    75
          commas_quote (map fst funvars) ^ " occur" ^ plural "s" "" funvars ^
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    76
          " in function position.", "Misspelled constructor???"]); true)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    77
      in
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    78
        (fname, length args)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    79
      end
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    80
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    81
    val grouped_args = AList.group (op =) (map check eqs)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    82
    val _ = grouped_args
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    83
      |> map (fn (fname, ars) =>
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    84
        length (distinct (op =) ars) = 1
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    85
        orelse error ("Function " ^ quote fname ^
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    86
          " has different numbers of arguments in different equations"))
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    87
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    88
    val not_defined = subtract (op =) (map fst grouped_args) fnames
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    89
    val _ = null not_defined
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    90
      orelse error ("No defining equations for function" ^
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    91
        plural " " "s " not_defined ^ commas_quote not_defined)
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    92
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    93
    fun check_sorts ((fname, fT), _) =
3045
d0ad264f8c4f updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents: 2999
diff changeset
    94
      Sorts.of_sort (Sign.classes_of (Proof_Context.theory_of ctxt)) (fT, @{sort "pt"})
2752
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    95
      orelse error (cat_lines
2860
25a7f421a3ba added a test that every function must be of pt-sort
Christian Urban <urbanc@in.tum.de>
parents: 2821
diff changeset
    96
      ["Type of " ^ quote fname ^ " is not of sort " ^ quote "pt" ^ ":",
2752
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    97
       Syntax.string_of_typ (Config.put show_sorts true ctxt) fT])
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    98
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
    99
    val _ = map check_sorts fixes
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   100
  in
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   101
    ()
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   102
  end
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   103
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   104
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   105
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   106
val simp_attribs = map (Attrib.internal o K)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   107
  [Simplifier.simp_add,
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   108
   Code.add_default_eqn_attribute,
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   109
   Nitpick_Simps.add]
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   110
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   111
val psimp_attribs = map (Attrib.internal o K)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   112
  [Nitpick_Psimps.add]
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   113
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   114
fun mk_defname fixes = fixes |> map (fst o fst) |> space_implode "_"
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   115
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   116
fun add_simps fnames post sort extra_qualify label mod_binding moreatts
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   117
  simps lthy =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   118
  let
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   119
    val spec = post simps
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   120
      |> map (apfst (apsnd (fn ats => moreatts @ ats)))
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   121
      |> map (apfst (apfst extra_qualify))
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   122
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   123
    val (saved_spec_simps, lthy) =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   124
      fold_map Local_Theory.note spec lthy
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   125
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   126
    val saved_simps = maps snd saved_spec_simps
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   127
    val simps_by_f = sort saved_simps
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   128
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   129
    fun add_for_f fname simps =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   130
      Local_Theory.note
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   131
        ((mod_binding (Binding.qualify true fname (Binding.name label)), []), simps)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   132
      #> snd
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   133
  in
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   134
    (saved_simps, fold2 add_for_f fnames simps_by_f lthy)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   135
  end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   136
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   137
(* nominal *)
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   138
fun prepare_nominal_function do_print prep default_constraint fixspec eqns config lthy =
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   139
  let
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   140
    val constrn_fxs = map (fn (b, T, mx) => (b, SOME (the_default default_constraint T), mx))
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   141
    val ((fixes0, spec0), ctxt') = prep (constrn_fxs fixspec) eqns lthy
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   142
    val fixes = map (apfst (apfst Binding.name_of)) fixes0;
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   143
    val spec = map (fn (bnd, prop) => (bnd, [prop])) spec0;
2789
32979078bfe9 functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents: 2752
diff changeset
   144
    val (eqs, post, sort_cont, cnames) =  
3203
01a13904aaa5 adapted to latest change of Markus on the function package
Christian Urban <urbanc@in.tum.de>
parents: 3190
diff changeset
   145
      empty_preproc nominal_check_defs (Function_Common.default_config) ctxt' fixes spec (* nominal *)
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   146
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   147
    val defname = mk_defname fixes
2860
25a7f421a3ba added a test that every function must be of pt-sort
Christian Urban <urbanc@in.tum.de>
parents: 2821
diff changeset
   148
    val NominalFunctionConfig {partials, ...} = config
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   149
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   150
    val ((goal_state, cont), lthy') =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   151
      Nominal_Function_Mutual.prepare_nominal_function_mutual config defname fixes eqs lthy
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   152
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   153
    fun afterqed [[proof]] lthy =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   154
      let
2973
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
   155
        val NominalFunctionResult {fs, R, psimps, simple_pinducts,
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
   156
          termination, domintros, cases, eqvts, ...} =
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   157
          cont (Thm.close_derivation proof)
2973
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
   158
  
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   159
        val fnames = map (fst o fst) fixes
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   160
        fun qualify n = Binding.name n
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   161
          |> Binding.qualify true defname
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   162
        val conceal_partial = if partials then I else Binding.conceal
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   163
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   164
        val addsmps = add_simps fnames post sort_cont
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   165
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   166
        val (((psimps', pinducts'), (_, [termination'])), lthy) =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   167
          lthy
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   168
          |> addsmps (conceal_partial o Binding.qualify false "partial")
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   169
               "psimps" conceal_partial psimp_attribs psimps
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   170
          ||>> Local_Theory.note ((conceal_partial (qualify "pinduct"),
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   171
                 [Attrib.internal (K (Rule_Cases.case_names cnames)),
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   172
                  Attrib.internal (K (Rule_Cases.consumes 1)),
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   173
                  Attrib.internal (K (Induct.induct_pred ""))]), simple_pinducts)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   174
          ||>> Local_Theory.note ((Binding.conceal (qualify "termination"), []), [termination])
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   175
          ||> (snd o Local_Theory.note ((qualify "cases",
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   176
                 [Attrib.internal (K (Rule_Cases.case_names cnames))]), [cases]))
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   177
          ||> (case domintros of NONE => I | SOME thms => 
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   178
                   Local_Theory.note ((qualify "domintros", []), thms) #> snd)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   179
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   180
        val info = { add_simps=addsmps, case_names=cnames, psimps=psimps',
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   181
          pinducts=snd pinducts', simps=NONE, inducts=NONE, termination=termination',
2973
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
   182
          fs=fs, R=R, defname=defname, is_partial=true, eqvts=eqvts}
d1038e67923a added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents: 2862
diff changeset
   183
3234
08c3ef07cef7 changes from upstream
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 3233
diff changeset
   184
        val _ = Proof_Display.print_consts do_print
3233
9ae285ce814e updated changes from upstream (AFP)
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 3231
diff changeset
   185
          (Position.thread_data ()) lthy (K false) (map fst fixes)
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   186
      in
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   187
        (info, 
3045
d0ad264f8c4f updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents: 2999
diff changeset
   188
         lthy |> Local_Theory.declaration {syntax = false, pervasive = false} 
d0ad264f8c4f updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents: 2999
diff changeset
   189
           (add_function_data o morph_function_data info))
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   190
      end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   191
  in
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   192
    ((goal_state, afterqed), lthy')
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   193
  end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   194
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   195
fun gen_add_nominal_function do_print prep default_constraint fixspec eqns config tac lthy =
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   196
  let
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   197
    val ((goal_state, afterqed), lthy') =
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   198
      prepare_nominal_function do_print prep default_constraint fixspec eqns config lthy
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   199
    val pattern_thm =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   200
      case SINGLE (tac lthy') goal_state of
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   201
        NONE => error "pattern completeness and compatibility proof failed"
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   202
      | SOME st => Goal.finish lthy' st
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   203
  in
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   204
    lthy'
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   205
    |> afterqed [[pattern_thm]]
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   206
  end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   207
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   208
val add_nominal_function =
3231
188826f1ccdb updated to massive changes in Isabelle
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 3227
diff changeset
   209
  gen_add_nominal_function false Specification.check_spec (Type_Infer.anyT @{sort type})
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   210
fun add_nominal_function_cmd a b c d int = 
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   211
  gen_add_nominal_function int Specification.read_spec "_::type" a b c d
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   212
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   213
fun gen_nominal_function do_print prep default_constraint fixspec eqns config lthy =
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   214
  let
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   215
    val ((goal_state, afterqed), lthy') =
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   216
      prepare_nominal_function do_print prep default_constraint fixspec eqns config lthy
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   217
  in
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   218
    lthy'
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   219
    |> Proof.theorem NONE (snd oo afterqed) [[(Logic.unprotect (concl_of goal_state), [])]]
3227
35bb5b013f0e updated with current AFP version
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 3203
diff changeset
   220
    |> Proof.refine (Method.primitive_text (K (K goal_state))) |> Seq.hd
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   221
  end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   222
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   223
val nominal_function =
3231
188826f1ccdb updated to massive changes in Isabelle
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 3227
diff changeset
   224
  gen_nominal_function false Specification.check_spec (Type_Infer.anyT @{sort type})
2992
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   225
fun nominal_function_cmd a b c int = 
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   226
  gen_nominal_function int Specification.read_spec "_::type" a b c
782a2cd1a8d0 made same changes as in main branch
Christian Urban <urbanc@in.tum.de>
parents: 2988
diff changeset
   227
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   228
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   229
fun add_case_cong n thy =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   230
  let
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   231
    val cong = #case_cong (Datatype.the_info thy n)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   232
      |> safe_mk_meta_eq
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   233
  in
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   234
    Context.theory_map
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   235
      (Function_Ctx_Tree.map_function_congs (Thm.add_thm cong)) thy
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   236
  end
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   237
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   238
val setup_case_cong = Datatype.interpretation (K (fold add_case_cong))
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   239
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   240
2752
9f44608ea28d changed default preprocessor that does not catch variables only occuring on the right
Christian Urban <urbanc@in.tum.de>
parents: 2745
diff changeset
   241
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   242
(* setup *)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   243
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   244
val setup =
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   245
  Attrib.setup @{binding fundef_cong}
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   246
    (Attrib.add_del Function_Ctx_Tree.cong_add Function_Ctx_Tree.cong_del)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   247
    "declaration of congruence rule for function definitions"
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   248
  #> setup_case_cong
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   249
  #> Function_Common.Termination_Simps.setup
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   250
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   251
val get_congs = Function_Ctx_Tree.get_function_congs
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   252
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   253
fun get_info ctxt t = Item_Net.retrieve (get_function ctxt) t
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   254
  |> the_single |> snd
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   255
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   256
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   257
(* outer syntax *)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   258
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   259
local
2999
68c894c513f6 updated to Isabelle 28 Aug
Christian Urban <urbanc@in.tum.de>
parents: 2992
diff changeset
   260
  val option_parser = Parse.group (fn () => "option")
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   261
    ((Parse.reserved "sequential" >> K Sequential)
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   262
     || ((Parse.reserved "default" |-- Parse.term) >> Default)
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   263
     || (Parse.reserved "domintros" >> K DomIntros)
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   264
     || (Parse.reserved "no_partials" >> K No_Partials)
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   265
     || ((Parse.reserved "invariant" |-- Parse.term) >> Invariant))
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   266
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   267
  fun config_parser default =
3234
08c3ef07cef7 changes from upstream
Christian Urban <christian dot urban at kcl dot ac dot uk>
parents: 3233
diff changeset
   268
    (Scan.optional (@{keyword "("} |-- Parse.!!! (Parse.list1 option_parser) --| @{keyword ")"}) [])
2819
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   269
     >> (fn opts => fold apply_opt opts default)
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   270
in
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   271
  fun nominal_function_parser default_cfg =
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   272
      config_parser default_cfg -- Parse.fixes -- Parse_Spec.where_alt_specs
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   273
end
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   274
4bd584ff4fab added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents: 2789
diff changeset
   275
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   276
(* nominal *)
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   277
val _ =
3190
1b7c034c9e9e used ML-antiquotation command_spec for new commands
Christian Urban <urbanc@in.tum.de>
parents: 3165
diff changeset
   278
  Outer_Syntax.local_theory_to_proof' @{command_spec "nominal_primrec"}
3135
92b9b8d2888d updated to new Isabelle (20 March)
Christian Urban <urbanc@in.tum.de>
parents: 3045
diff changeset
   279
    "define general recursive nominal functions"
92b9b8d2888d updated to new Isabelle (20 March)
Christian Urban <urbanc@in.tum.de>
parents: 3045
diff changeset
   280
       (nominal_function_parser nominal_default_config
92b9b8d2888d updated to new Isabelle (20 March)
Christian Urban <urbanc@in.tum.de>
parents: 3045
diff changeset
   281
          >> (fn ((config, fixes), statements) => nominal_function_cmd fixes statements config))
2665
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   282
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   283
16b5a67ee279 exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   284
end