| author | blanchet | 
| Thu, 09 Jan 2014 14:09:44 +0100 | |
| changeset 54950 | f00012c20344 | 
| parent 54601 | 91a1e4aa7c80 | 
| child 54960 | d72279b9bc44 | 
| permissions | -rw-r--r-- | 
| 54601 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 1 | (* Title: HOL/BNF/Tools/bnf_decl.ML | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 2 | Author: Dmitriy Traytel, TU Muenchen | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 3 | Copyright 2013 | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 4 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 5 | Axiomatic declaration of bounded natural functors. | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 6 | *) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 7 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 8 | signature BNF_DECL = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 9 | sig | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 10 | val bnf_decl: (binding option * (typ * sort)) list -> binding -> mixfix -> binding -> binding -> | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 11 | local_theory -> BNF_Def.bnf * local_theory | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 12 | end | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 13 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 14 | structure BNF_Decl : BNF_DECL = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 15 | struct | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 16 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 17 | open BNF_Util | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 18 | open BNF_Def | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 19 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 20 | fun prepare_decl prepare_constraint prepare_typ raw_vars b mx user_mapb user_relb lthy = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 21 | let | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 22 | fun prepare_type_arg (set_opt, (ty, c)) = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 23 | let val s = fst (dest_TFree (prepare_typ lthy ty)) in | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 24 | (set_opt, (s, prepare_constraint lthy c)) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 25 | end; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 26 | val ((user_setbs, vars), raw_vars') = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 27 | map prepare_type_arg raw_vars | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 28 | |> `split_list | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 29 | |>> apfst (map_filter I); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 30 | val deads = map_filter (fn (NONE, x) => SOME x | _ => NONE) raw_vars'; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 31 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 32 | fun mk_b name user_b = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 33 | (if Binding.is_empty user_b then Binding.prefix_name (name ^ "_") b else user_b) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 34 | |> Binding.qualify false (Binding.name_of b); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 35 | val (Tname, lthy) = Typedecl.basic_typedecl (b, length vars, mx) lthy; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 36 | val (bd_type_Tname, lthy) = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 37 | Typedecl.basic_typedecl (mk_b "bd_type" Binding.empty, length deads, NoSyn) lthy; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 38 | val T = Type (Tname, map TFree vars); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 39 | val bd_type_T = Type (bd_type_Tname, map TFree deads); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 40 | val lives = map TFree (filter_out (member (op =) deads) vars); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 41 | val live = length lives; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 42 | val _ = "Trying to declare a BNF with no live variables" |> null lives ? error; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 43 | val (lives', _) = BNF_Util.mk_TFrees (length lives) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 44 | (fold Variable.declare_typ (map TFree vars) lthy); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 45 | val T' = Term.typ_subst_atomic (lives ~~ lives') T; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 46 | val mapT = map2 (curry op -->) lives lives' ---> T --> T'; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 47 | val setTs = map (fn U => T --> HOLogic.mk_setT U) lives; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 48 | val bdT = BNF_Util.mk_relT (bd_type_T, bd_type_T); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 49 | val mapb = mk_b BNF_Def.mapN user_mapb; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 50 | val bdb = mk_b "bd" Binding.empty; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 51 | val setbs = map2 (fn b => fn i => mk_b (BNF_Def.mk_setN i) b) user_setbs | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 52 | (if live = 1 then [0] else 1 upto live); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 53 | val lthy = Local_Theory.background_theory | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 54 | (Sign.add_consts_i ((mapb, mapT, NoSyn) :: (bdb, bdT, NoSyn) :: | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 55 | map2 (fn b => fn T => (b, T, NoSyn)) setbs setTs)) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 56 | lthy; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 57 | val Fmap = Const (Local_Theory.full_name lthy mapb, mapT); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 58 | val Fsets = map2 (fn setb => fn setT => | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 59 | Const (Local_Theory.full_name lthy setb, setT)) setbs setTs; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 60 | val Fbd = Const (Local_Theory.full_name lthy bdb, bdT); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 61 | val (key, goals, (triv_tac_opt, wit_goalss), after_qed, lthy, _) = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 62 | prepare_def Do_Inline (user_policy Note_Some) I (K I) (K I) (SOME (map TFree deads)) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 63 | user_mapb user_relb user_setbs ((((((Binding.empty, T), Fmap), Fsets), Fbd), []), NONE) lthy; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 64 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 65 | fun mk_wits_tac set_maps = K (TRYALL Goal.conjunction_tac) THEN' the triv_tac_opt set_maps; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 66 | val wit_goals = map Logic.mk_conjunction_balanced wit_goalss; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 67 | fun mk_wit_thms set_maps = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 68 | Goal.prove_sorry lthy [] [] (Logic.mk_conjunction_balanced wit_goals) (mk_wits_tac set_maps) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 69 | |> Conjunction.elim_balanced (length wit_goals) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 70 | |> map2 (Conjunction.elim_balanced o length) wit_goalss | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 71 | |> map (map (Thm.close_derivation o Thm.forall_elim_vars 0)); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 72 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 73 | val ((_, [thms]), (lthy_old, lthy)) = Local_Theory.background_theory_result | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 74 | (Specification.axiomatization [] [((mk_b "axioms" Binding.empty, []), goals)]) lthy | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 75 | ||> `Local_Theory.restore; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 76 | val phi = Proof_Context.export_morphism lthy_old lthy; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 77 | in | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 78 | BNF_Def.register_bnf key (after_qed mk_wit_thms (map single (Morphism.fact phi thms)) lthy) | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 79 | end; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 80 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 81 | val bnf_decl = prepare_decl (K I) (K I); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 82 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 83 | fun read_constraint _ NONE = HOLogic.typeS | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 84 | | read_constraint ctxt (SOME s) = Syntax.read_sort ctxt s; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 85 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 86 | val bnf_decl_cmd = prepare_decl read_constraint Syntax.parse_typ; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 87 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 88 | val parse_bnf_decl = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 89 | parse_type_args_named_constrained -- parse_binding -- parse_map_rel_bindings -- Parse.opt_mixfix; | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 90 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 91 | val _ = | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 92 |   Outer_Syntax.local_theory @{command_spec "bnf_decl"} "bnf declaration"
 | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 93 | (parse_bnf_decl >> | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 94 | (fn (((bsTs, b), (mapb, relb)), mx) => bnf_decl_cmd bsTs b mx mapb relb #> snd)); | 
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 95 | |
| 
91a1e4aa7c80
command for axiomatic declaration of bnfs---allow theoreticians to fix an arbitrary type with functorial structure and work abstractly on it
 traytel parents: diff
changeset | 96 | end; |