| author | blanchet | 
| Wed, 01 Sep 2010 18:47:07 +0200 | |
| changeset 39000 | d73a054e018c | 
| parent 38756 | d07959fabde6 | 
| child 39557 | fe5722fce758 | 
| permissions | -rw-r--r-- | 
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
30364diff
changeset | 1 | (* Title: HOL/Tools/choice_specification.ML | 
| 14115 | 2 | Author: Sebastian Skalberg, TU Muenchen | 
| 3 | ||
| 4 | Package for defining constants by specification. | |
| 5 | *) | |
| 6 | ||
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
30364diff
changeset | 7 | signature CHOICE_SPECIFICATION = | 
| 14115 | 8 | sig | 
| 35807 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 9 | val close_form : term -> term | 
| 18729 | 10 | val add_specification: string option -> (bstring * xstring * bool) list -> | 
| 11 | theory * thm -> theory * thm | |
| 14115 | 12 | end | 
| 13 | ||
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
30364diff
changeset | 14 | structure Choice_Specification: CHOICE_SPECIFICATION = | 
| 14115 | 15 | struct | 
| 16 | ||
| 26478 | 17 | (* actual code *) | 
| 14115 | 18 | |
| 35807 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 19 | fun close_form t = | 
| 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 20 | fold_rev (fn (s, T) => fn t => HOLogic.mk_all (s, T, t)) | 
| 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 21 | (map dest_Free (OldTerm.term_frees t)) t | 
| 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 22 | |
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 23 | local | 
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 24 | fun mk_definitional [] arg = arg | 
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 25 | | mk_definitional ((thname,cname,covld)::cos) (thy,thm) = | 
| 17336 | 26 | case HOLogic.dest_Trueprop (concl_of thm) of | 
| 38558 | 27 |             Const(@{const_name Ex},_) $ P =>
 | 
| 17336 | 28 | let | 
| 29 | val ctype = domain_type (type_of P) | |
| 22578 | 30 | val cname_full = Sign.intern_const thy cname | 
| 17336 | 31 | val cdefname = if thname = "" | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30280diff
changeset | 32 | then Thm.def_name (Long_Name.base_name cname) | 
| 17336 | 33 | else thname | 
| 34 | val def_eq = Logic.mk_equals (Const(cname_full,ctype), | |
| 35 | HOLogic.choice_const ctype $ P) | |
| 29579 | 36 | val (thms, thy') = PureThy.add_defs covld [((Binding.name cdefname, def_eq),[])] thy | 
| 26478 | 37 |                 val thm' = [thm,hd thms] MRS @{thm exE_some}
 | 
| 17336 | 38 | in | 
| 39 | mk_definitional cos (thy',thm') | |
| 40 | end | |
| 41 |           | _ => raise THM ("Internal error: Bad specification theorem",0,[thm])
 | |
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 42 | |
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 43 | fun mk_axiomatic axname cos arg = | 
| 17336 | 44 | let | 
| 45 | fun process [] (thy,tm) = | |
| 46 | let | |
| 35897 
8758895ea413
eliminated old-style Drule.add_axiom in favour of Specification.axiom, with explicit Drule.export_without_context to imitate the old behaviour;
 wenzelm parents: 
35856diff
changeset | 47 | val (thm, thy') = | 
| 
8758895ea413
eliminated old-style Drule.add_axiom in favour of Specification.axiom, with explicit Drule.export_without_context to imitate the old behaviour;
 wenzelm parents: 
35856diff
changeset | 48 | Specification.axiom ((Binding.name axname, []), HOLogic.mk_Trueprop tm) thy | 
| 17336 | 49 | in | 
| 35897 
8758895ea413
eliminated old-style Drule.add_axiom in favour of Specification.axiom, with explicit Drule.export_without_context to imitate the old behaviour;
 wenzelm parents: 
35856diff
changeset | 50 | (thy', Drule.export_without_context thm) | 
| 17336 | 51 | end | 
| 52 | | process ((thname,cname,covld)::cos) (thy,tm) = | |
| 53 | case tm of | |
| 38558 | 54 |                     Const(@{const_name Ex},_) $ P =>
 | 
| 17336 | 55 | let | 
| 56 | val ctype = domain_type (type_of P) | |
| 22578 | 57 | val cname_full = Sign.intern_const thy cname | 
| 17336 | 58 | val cdefname = if thname = "" | 
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30280diff
changeset | 59 | then Thm.def_name (Long_Name.base_name cname) | 
| 17336 | 60 | else thname | 
| 61 | val co = Const(cname_full,ctype) | |
| 62 | val thy' = Theory.add_finals_i covld [co] thy | |
| 63 | val tm' = case P of | |
| 64 | Abs(_, _, bodt) => subst_bound (co, bodt) | |
| 65 | | _ => P $ co | |
| 66 | in | |
| 67 | process cos (thy',tm') | |
| 68 | end | |
| 69 |                   | _ => raise TERM ("Internal error: Bad specification theorem",[tm])
 | |
| 70 | in | |
| 71 | process cos arg | |
| 72 | end | |
| 14115 | 73 | |
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 74 | in | 
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 75 | fun proc_exprop axiomatic cos arg = | 
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 76 | case axiomatic of | 
| 17336 | 77 | SOME axname => mk_axiomatic axname cos (apsnd (HOLogic.dest_Trueprop o concl_of) arg) | 
| 15531 | 78 | | NONE => mk_definitional cos arg | 
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 79 | end | 
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 80 | |
| 36618 
7a0990473e03
specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result;
 wenzelm parents: 
36615diff
changeset | 81 | fun add_specification axiomatic cos = | 
| 
7a0990473e03
specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result;
 wenzelm parents: 
36615diff
changeset | 82 | proc_exprop axiomatic cos | 
| 
7a0990473e03
specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result;
 wenzelm parents: 
36615diff
changeset | 83 | #> apsnd Drule.export_without_context | 
| 14115 | 84 | |
| 18729 | 85 | |
| 14115 | 86 | (* Collect all intances of constants in term *) | 
| 87 | ||
| 88 | fun collect_consts ( t $ u,tms) = collect_consts (u,collect_consts (t,tms)) | |
| 89 | | collect_consts ( Abs(_,_,t),tms) = collect_consts (t,tms) | |
| 18921 | 90 | | collect_consts (tm as Const _,tms) = insert (op aconv) tm tms | 
| 14115 | 91 | | collect_consts ( _,tms) = tms | 
| 92 | ||
| 35845 
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
 wenzelm parents: 
35807diff
changeset | 93 | (* Complementing Type.varify_global... *) | 
| 14115 | 94 | |
| 35845 
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
 wenzelm parents: 
35807diff
changeset | 95 | fun unvarify_global t fmap = | 
| 14115 | 96 | let | 
| 17336 | 97 | val fmap' = map Library.swap fmap | 
| 17377 | 98 | fun unthaw (f as (a, S)) = | 
| 99 | (case AList.lookup (op =) fmap' a of | |
| 17336 | 100 | NONE => TVar f | 
| 17377 | 101 | | SOME (b, _) => TFree (b, S)) | 
| 14115 | 102 | in | 
| 20548 
8ef25fe585a8
renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
 wenzelm parents: 
20344diff
changeset | 103 | map_types (map_type_tvar unthaw) t | 
| 14115 | 104 | end | 
| 105 | ||
| 106 | (* The syntactic meddling needed to setup add_specification for work *) | |
| 107 | ||
| 17336 | 108 | fun process_spec axiomatic cos alt_props thy = | 
| 14115 | 109 | let | 
| 17336 | 110 | fun zip3 [] [] [] = [] | 
| 111 | | zip3 (x::xs) (y::ys) (z::zs) = (x,y,z)::zip3 xs ys zs | |
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
30364diff
changeset | 112 | | zip3 _ _ _ = error "Choice_Specification.process_spec internal error" | 
| 14167 | 113 | |
| 17336 | 114 | fun myfoldr f [x] = x | 
| 115 | | myfoldr f (x::xs) = f (x,myfoldr f xs) | |
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
30364diff
changeset | 116 | | myfoldr f [] = error "Choice_Specification.process_spec internal error" | 
| 14164 
8c3fab596219
Allowed for splitting the specification over several lemmas.
 skalberg parents: 
14122diff
changeset | 117 | |
| 17895 | 118 | val rew_imps = alt_props |> | 
| 35625 | 119 | map (Object_Logic.atomize o Thm.cterm_of thy o Syntax.read_prop_global thy o snd) | 
| 17895 | 120 | val props' = rew_imps |> | 
| 22902 
ac833b4bb7ee
moved some Drule operations to Thm (see more_thm.ML);
 wenzelm parents: 
22709diff
changeset | 121 | map (HOLogic.dest_Trueprop o term_of o snd o Thm.dest_equals o cprop_of) | 
| 14166 | 122 | |
| 17336 | 123 | fun proc_single prop = | 
| 124 | let | |
| 29265 
5b4247055bd7
moved old add_term_vars, add_term_frees etc. to structure OldTerm;
 wenzelm parents: 
29006diff
changeset | 125 | val frees = OldTerm.term_frees prop | 
| 21858 
05f57309170c
avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
 wenzelm parents: 
21434diff
changeset | 126 | val _ = forall (fn v => Sign.of_sort thy (type_of v,HOLogic.typeS)) frees | 
| 
05f57309170c
avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
 wenzelm parents: 
21434diff
changeset | 127 | orelse error "Specificaton: Only free variables of sort 'type' allowed" | 
| 35807 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 128 | val prop_closed = close_form prop | 
| 17336 | 129 | in | 
| 130 | (prop_closed,frees) | |
| 131 | end | |
| 14166 | 132 | |
| 17336 | 133 | val props'' = map proc_single props' | 
| 134 | val frees = map snd props'' | |
| 135 | val prop = myfoldr HOLogic.mk_conj (map fst props'') | |
| 17895 | 136 | val cprop = cterm_of thy (HOLogic.mk_Trueprop prop) | 
| 14164 
8c3fab596219
Allowed for splitting the specification over several lemmas.
 skalberg parents: 
14122diff
changeset | 137 | |
| 35845 
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
 wenzelm parents: 
35807diff
changeset | 138 | val (vmap, prop_thawed) = Type.varify_global [] prop | 
| 17336 | 139 | val thawed_prop_consts = collect_consts (prop_thawed,[]) | 
| 140 | val (altcos,overloaded) = Library.split_list cos | |
| 141 | val (names,sconsts) = Library.split_list altcos | |
| 24707 | 142 | val consts = map (Syntax.read_term_global thy) sconsts | 
| 21858 
05f57309170c
avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
 wenzelm parents: 
21434diff
changeset | 143 | val _ = not (Library.exists (not o Term.is_Const) consts) | 
| 
05f57309170c
avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
 wenzelm parents: 
21434diff
changeset | 144 | orelse error "Specification: Non-constant found as parameter" | 
| 14166 | 145 | |
| 17336 | 146 | fun proc_const c = | 
| 147 | let | |
| 35845 
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
 wenzelm parents: 
35807diff
changeset | 148 | val (_, c') = Type.varify_global [] c | 
| 17336 | 149 | val (cname,ctyp) = dest_Const c' | 
| 150 | in | |
| 33317 | 151 | case filter (fn t => let val (name,typ) = dest_Const t | 
| 19414 | 152 | in name = cname andalso Sign.typ_equiv thy (typ, ctyp) | 
| 17336 | 153 | end) thawed_prop_consts of | 
| 26939 
1035c89b4c02
moved global pretty/string_of functions from Sign to Syntax;
 wenzelm parents: 
26928diff
changeset | 154 |                     [] => error ("Specification: No suitable instances of constant \"" ^ Syntax.string_of_term_global thy c ^ "\" found")
 | 
| 35845 
e5980f0ad025
renamed varify/unvarify operations to varify_global/unvarify_global to emphasize that these only work in a global situation;
 wenzelm parents: 
35807diff
changeset | 155 | | [cf] => unvarify_global cf vmap | 
| 26939 
1035c89b4c02
moved global pretty/string_of functions from Sign to Syntax;
 wenzelm parents: 
26928diff
changeset | 156 |                   | _ => error ("Specification: Several variations of \"" ^ Syntax.string_of_term_global thy c ^ "\" found (try applying explicit type constraints)")
 | 
| 17336 | 157 | end | 
| 158 | val proc_consts = map proc_const consts | |
| 33339 | 159 | fun mk_exist c prop = | 
| 17336 | 160 | let | 
| 161 | val T = type_of c | |
| 30364 
577edc39b501
moved basic algebra of long names from structure NameSpace to Long_Name;
 wenzelm parents: 
30280diff
changeset | 162 | val cname = Long_Name.base_name (fst (dest_Const c)) | 
| 17336 | 163 | val vname = if Syntax.is_identifier cname | 
| 164 | then cname | |
| 165 | else "x" | |
| 166 | in | |
| 167 | HOLogic.exists_const T $ Abs(vname,T,Term.abstract_over (c,prop)) | |
| 168 | end | |
| 33339 | 169 | val ex_prop = fold_rev mk_exist proc_consts prop | 
| 17336 | 170 | val cnames = map (fst o dest_Const) proc_consts | 
| 171 | fun post_process (arg as (thy,thm)) = | |
| 172 | let | |
| 33245 | 173 | fun inst_all thy v thm = | 
| 17336 | 174 | let | 
| 17895 | 175 | val cv = cterm_of thy v | 
| 17336 | 176 | val cT = ctyp_of_term cv | 
| 177 | val spec' = instantiate' [SOME cT] [NONE,SOME cv] spec | |
| 178 | in | |
| 179 | thm RS spec' | |
| 180 | end | |
| 22578 | 181 | fun remove_alls frees thm = | 
| 33245 | 182 | fold (inst_all (Thm.theory_of_thm thm)) frees thm | 
| 17336 | 183 | fun process_single ((name,atts),rew_imp,frees) args = | 
| 184 | let | |
| 185 | fun undo_imps thm = | |
| 36945 | 186 | Thm.equal_elim (Thm.symmetric rew_imp) thm | 
| 14164 
8c3fab596219
Allowed for splitting the specification over several lemmas.
 skalberg parents: 
14122diff
changeset | 187 | |
| 18358 | 188 | fun add_final (arg as (thy, thm)) = | 
| 17336 | 189 | if name = "" | 
| 18358 | 190 | then arg |> Library.swap | 
| 32091 
30e2ffbba718
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
 wenzelm parents: 
31723diff
changeset | 191 |                             else (writeln ("  " ^ name ^ ": " ^ Display.string_of_thm_global thy thm);
 | 
| 29579 | 192 | PureThy.store_thm (Binding.name name, thm) thy) | 
| 17336 | 193 | in | 
| 194 | args |> apsnd (remove_alls frees) | |
| 195 | |> apsnd undo_imps | |
| 35021 
c839a4c670c6
renamed old-style Drule.standard to Drule.export_without_context, to emphasize that this is in no way a standard operation;
 wenzelm parents: 
33339diff
changeset | 196 | |> apsnd Drule.export_without_context | 
| 35807 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 197 | |> Thm.theory_attributes (map (Attrib.attribute thy) | 
| 
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
 blanchet parents: 
35625diff
changeset | 198 | (Attrib.internal (K Nitpick_Choice_Specs.add) :: atts)) | 
| 17336 | 199 | |> add_final | 
| 18358 | 200 | |> Library.swap | 
| 17336 | 201 | end | 
| 14164 
8c3fab596219
Allowed for splitting the specification over several lemmas.
 skalberg parents: 
14122diff
changeset | 202 | |
| 17336 | 203 | fun process_all [proc_arg] args = | 
| 204 | process_single proc_arg args | |
| 205 | | process_all (proc_arg::rest) (thy,thm) = | |
| 206 | let | |
| 207 | val single_th = thm RS conjunct1 | |
| 208 | val rest_th = thm RS conjunct2 | |
| 209 | val (thy',_) = process_single proc_arg (thy,single_th) | |
| 210 | in | |
| 211 | process_all rest (thy',rest_th) | |
| 212 | end | |
| 31723 
f5cafe803b55
discontinued ancient tradition to suffix certain ML module names with "_package"
 haftmann parents: 
30364diff
changeset | 213 | | process_all [] _ = error "Choice_Specification.process_spec internal error" | 
| 17336 | 214 | val alt_names = map fst alt_props | 
| 215 | val _ = if exists (fn(name,_) => not (name = "")) alt_names | |
| 216 | then writeln "specification" | |
| 217 | else () | |
| 218 | in | |
| 36618 
7a0990473e03
specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result;
 wenzelm parents: 
36615diff
changeset | 219 | arg |> apsnd Thm.unvarify_global | 
| 17336 | 220 | |> process_all (zip3 alt_names rew_imps frees) | 
| 221 | end | |
| 20903 | 222 | |
| 38756 
d07959fabde6
renamed ProofContext.theory(_result) to ProofContext.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
 wenzelm parents: 
38558diff
changeset | 223 | fun after_qed [[thm]] = ProofContext.background_theory (fn thy => | 
| 
d07959fabde6
renamed ProofContext.theory(_result) to ProofContext.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
 wenzelm parents: 
38558diff
changeset | 224 | #1 (post_process (add_specification axiomatic (zip3 names cnames overloaded) (thy, thm)))); | 
| 14115 | 225 | in | 
| 20903 | 226 | thy | 
| 36610 
bafd82950e24
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
 wenzelm parents: 
36323diff
changeset | 227 | |> ProofContext.init_global | 
| 36618 
7a0990473e03
specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result;
 wenzelm parents: 
36615diff
changeset | 228 | |> Variable.declare_term ex_prop | 
| 36323 
655e2d74de3a
modernized naming conventions of main Isar proof elements;
 wenzelm parents: 
35897diff
changeset | 229 | |> Proof.theorem NONE after_qed [[(HOLogic.mk_Trueprop ex_prop, [])]] | 
| 20903 | 230 | end; | 
| 14115 | 231 | |
| 17336 | 232 | |
| 14115 | 233 | (* outer syntax *) | 
| 234 | ||
| 36960 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 235 | val opt_name = Scan.optional (Parse.name --| Parse.$$$ ":") "" | 
| 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 236 | val opt_overloaded = Parse.opt_keyword "overloaded" | 
| 14116 
63337d8e6e0f
Added optional theorem names for the constant definitions added during
 skalberg parents: 
14115diff
changeset | 237 | |
| 14115 | 238 | val specification_decl = | 
| 36960 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 239 |   Parse.$$$ "(" |-- Scan.repeat1 (opt_name -- Parse.term -- opt_overloaded) --| Parse.$$$ ")" --
 | 
| 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 240 | Scan.repeat1 ((Parse_Spec.opt_thm_name ":" >> apfst Binding.name_of) -- Parse.prop) | 
| 14115 | 241 | |
| 24867 | 242 | val _ = | 
| 36960 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 243 | Outer_Syntax.command "specification" "define constants by specification" Keyword.thy_goal | 
| 14164 
8c3fab596219
Allowed for splitting the specification over several lemmas.
 skalberg parents: 
14122diff
changeset | 244 | (specification_decl >> (fn (cos,alt_props) => | 
| 17336 | 245 | Toplevel.print o (Toplevel.theory_to_proof | 
| 246 | (process_spec NONE cos alt_props)))) | |
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 247 | |
| 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 248 | val ax_specification_decl = | 
| 36960 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 249 | Parse.name -- | 
| 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 250 |     (Parse.$$$ "(" |-- Scan.repeat1 (opt_name -- Parse.term -- opt_overloaded) --| Parse.$$$ ")" --
 | 
| 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 251 | Scan.repeat1 ((Parse_Spec.opt_thm_name ":" >> apfst Binding.name_of) -- Parse.prop)) | 
| 14115 | 252 | |
| 24867 | 253 | val _ = | 
| 36960 
01594f816e3a
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
 wenzelm parents: 
36954diff
changeset | 254 | Outer_Syntax.command "ax_specification" "define constants by specification" Keyword.thy_goal | 
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 255 | (ax_specification_decl >> (fn (axname,(cos,alt_props)) => | 
| 17336 | 256 | Toplevel.print o (Toplevel.theory_to_proof | 
| 257 | (process_spec (SOME axname) cos alt_props)))) | |
| 14222 
1e61f23fd359
Added axiomatic specifications (ax_specification).
 skalberg parents: 
14167diff
changeset | 258 | |
| 14115 | 259 | end |