src/HOL/Tools/function_package/fundef_package.ML
author krauss
Mon, 31 Jul 2006 18:07:42 +0200
changeset 20270 3abe7dae681e
parent 19938 241a7777a3ff
child 20285 23f5cd23c1e1
permissions -rw-r--r--
Function package can now do automatic splits of overlapping datatype patterns


(*  Title:      HOL/Tools/function_package/fundef_package.ML
    ID:         $Id$
    Author:     Alexander Krauss, TU Muenchen

A package for general recursive function definitions. 
Isar commands.

*)

signature FUNDEF_PACKAGE = 
sig
    val add_fundef : ((bstring * (Attrib.src list * bool)) * string) list list -> bool -> theory -> Proof.state (* Need an _i variant *)

    val cong_add: attribute
    val cong_del: attribute
							 
    val setup : theory -> theory
    val get_congs : theory -> thm list
end


structure FundefPackage : FUNDEF_PACKAGE =
struct

open FundefCommon

val True_implies = thm "True_implies"


fun add_simps label moreatts (MutualPart {f_name, ...}, psimps) spec_part thy =
    let 
      val psimpss = Library.unflat (map snd spec_part) psimps
      val (names, attss) = split_list (map fst spec_part) 

      val thy = thy |> Theory.add_path f_name 
                
      val thy = thy |> Theory.add_path label
      val spsimpss = map (map standard) psimpss (* FIXME *)
      val add_list = (names ~~ spsimpss) ~~ attss
      val (_, thy) = PureThy.add_thmss add_list thy
      val thy = thy |> Theory.parent_path
                
      val (_, thy) = PureThy.add_thmss [((label, flat spsimpss), Simplifier.simp_add :: moreatts)] thy
      val thy = thy |> Theory.parent_path
    in
      thy
    end
    





fun fundef_afterqed congs mutual_info name data spec [[result]] thy =
    let
	val fundef_data = FundefMutual.mk_partial_rules_mutual thy mutual_info data result
	val FundefMResult {psimps, subset_pinducts, simple_pinducts, termination, domintros, cases, ...} = fundef_data
        val Mutual {parts, ...} = mutual_info

	val Prep {names = Names {acc_R=accR, ...}, ...} = data
	val dom_abbrev = Logic.mk_equals (Free (name ^ "_dom", fastype_of accR), accR)
	val (_, thy) = LocalTheory.mapping NONE (Specification.abbreviation_i ("", false) [(NONE, dom_abbrev)]) thy

        val thy = fold2 (add_simps "psimps" []) (parts ~~ psimps) spec thy

        val casenames = flat (map (map (fst o fst)) spec)

	val thy = thy |> Theory.add_path name
	val (_, thy) = PureThy.add_thms [(("cases", cases), [RuleCases.case_names casenames])] thy
	val (_, thy) = PureThy.add_thmss [(("domintros", domintros), [])] thy
	val (_, thy) = PureThy.add_thms [(("termination", standard termination), [])] thy
	val (_,thy) = PureThy.add_thmss [(("pinduct", map standard simple_pinducts), [RuleCases.case_names casenames, InductAttrib.induct_set ""])] thy
	val thy = thy |> Theory.parent_path
    in
      add_fundef_data name (fundef_data, mutual_info, spec) thy
    end

fun gen_add_fundef prep_att eqns_attss preprocess thy =
    let
      fun prep_eqns neqs =
          neqs
            |> map (apsnd (Sign.read_prop thy))    
            |> map (apfst (apsnd (apfst (map (prep_att thy)))))
            |> FundefSplit.split_some_equations (ProofContext.init thy)
      
      val spec = map prep_eqns eqns_attss
      val t_eqnss = map (flat o map snd) spec

(*
 val t_eqns = if preprocess then map (FundefSplit.split_all_equations (ProofContext.init thy)) t_eqns
              else t_eqns
*)

      val congs = get_fundef_congs (Context.Theory thy)

      val (mutual_info, name, (data, thy)) = FundefMutual.prepare_fundef_mutual congs t_eqnss thy
      val Prep {goal, goalI, ...} = data
    in
	thy |> ProofContext.init
	    |> Proof.theorem_i PureThy.internalK NONE (fundef_afterqed congs mutual_info name data spec) NONE ("", [])
	    [(("", []), [(goal, [])])]
            |> Proof.refine (Method.primitive_text (fn _ => goalI))
            |> Seq.hd
    end


fun total_termination_afterqed name (Mutual {parts, ...}) thmss thy =
    let
	val totality = hd (hd thmss)

	val (FundefMResult {psimps, simple_pinducts, ... }, Mutual {parts, ...}, spec)
	  = the (get_fundef_data name thy)

	val remove_domain_condition = full_simplify (HOL_basic_ss addsimps [totality, True_implies])

	val tsimps = map (map remove_domain_condition) psimps
	val tinduct = map remove_domain_condition simple_pinducts

        val has_guards = exists ((fn (Const ("Trueprop", _) $ _) => false | _ => true) o prop_of) (flat tsimps)
        val allatts = if has_guards then [] else [RecfunCodegen.add NONE]

        val thy = fold2 (add_simps "simps" allatts) (parts ~~ tsimps) spec thy

	val thy = Theory.add_path name thy
		  
	val (_, thy) = PureThy.add_thmss [(("induct", map standard tinduct), [])] thy 
	val thy = Theory.parent_path thy
    in
	thy
    end

(*
fun mk_partial_rules name D_name D domT idomT thmss thy =
    let
	val [subs, dcl] = (hd thmss)

	val {f_const, f_curried_const, G_const, R_const, G_elims, completeness, f_simps, names_attrs, subset_induct, ... }
	  = the (Symtab.lookup (FundefData.get thy) name)

	val D_implies_dom = subs COMP (instantiate' [SOME (ctyp_of thy idomT)] 
						    [SOME (cterm_of thy D)]
						    subsetD)

	val D_simps = map (curry op RS D_implies_dom) f_simps

	val D_induct = subset_induct
			   |> cterm_instantiate [(cterm_of thy (Var (("D",0), fastype_of D)) ,cterm_of thy D)]
			   |> curry op COMP subs
			   |> curry op COMP (dcl |> forall_intr (cterm_of thy (Var (("z",0), idomT)))
						 |> forall_intr (cterm_of thy (Var (("x",0), idomT))))

	val ([tinduct'], thy2) = PureThy.add_thms [((name ^ "_" ^ D_name ^ "_induct", D_induct), [])] thy
	val ([tsimps'], thy3) = PureThy.add_thmss [((name ^ "_" ^ D_name ^ "_simps", D_simps), [])] thy2
    in
	thy3
    end
*)
 

fun fundef_setup_termination_proof name NONE thy = 
    let
	val name = if name = "" then get_last_fundef thy else name
	val data = the (get_fundef_data name thy)
                   handle Option.Option => raise ERROR ("No such function definition: " ^ name)

	val (res as FundefMResult {termination, ...}, mutual, _) = data
	val goal = FundefTermination.mk_total_termination_goal data
    in
	thy |> ProofContext.init
	    |> ProofContext.note_thmss_i [(("termination", 
					    [ContextRules.intro_query NONE]), [([standard termination], [])])] |> snd
	    |> Proof.theorem_i PureThy.internalK NONE (total_termination_afterqed name mutual) NONE ("", [])
	    [(("", []), [(goal, [])])]
    end	
  | fundef_setup_termination_proof name (SOME (dom_name, dom)) thy =
    let
	val name = if name = "" then get_last_fundef thy else name
	val data = the (get_fundef_data name thy)
	val (subs, dcl) = FundefTermination.mk_partial_termination_goal thy data dom
    in
	thy |> ProofContext.init
	    |> Proof.theorem_i PureThy.internalK NONE (K I) NONE ("", [])
	    [(("", []), [(subs, []), (dcl, [])])]
    end	


val add_fundef = gen_add_fundef Attrib.attribute



(* congruence rules *)

val cong_add = Thm.declaration_attribute (map_fundef_congs o Drule.add_rule o safe_mk_meta_eq);
val cong_del = Thm.declaration_attribute (map_fundef_congs o Drule.del_rule o safe_mk_meta_eq);


(* setup *)

val setup = FundefData.init #> FundefCongs.init 
	#>  Attrib.add_attributes
		[("fundef_cong", Attrib.add_del_args cong_add cong_del, "declaration of congruence rule for function definitions")]


val get_congs = FundefCommon.get_fundef_congs o Context.Theory


(* outer syntax *)

local structure P = OuterParse and K = OuterKeyword in



val star = Scan.one (fn t => (OuterLex.val_of t = "*"));


val attribs_with_star = P.$$$ "[" |-- P.!!! ((P.list (star >> K NONE || P.attrib >> SOME)) 
                                               >> (fn x => (map_filter I x, exists is_none x)))
                              --| P.$$$ "]";

val opt_attribs_with_star = Scan.optional attribs_with_star ([], false);

fun opt_thm_name_star s =
  Scan.optional ((P.name -- opt_attribs_with_star || (attribs_with_star >> pair "")) --| P.$$$ s) ("", ([], false));


val function_decl =
    Scan.repeat1 (opt_thm_name_star ":" -- P.prop);

val functionP =
  OuterSyntax.command "function" "define general recursive functions" K.thy_goal
  (((Scan.optional (P.$$$ "(" -- P.!!! (P.$$$ "pre" -- P.$$$ ")") >> K true) false) --    
  P.and_list1 function_decl) >> (fn (prepr, eqnss) =>
                                    Toplevel.print o Toplevel.theory_to_proof (add_fundef eqnss prepr)));

val terminationP =
  OuterSyntax.command "termination" "prove termination of a recursive function" K.thy_goal
  ((Scan.optional P.name "" -- Scan.option (P.$$$ "(" |-- Scan.optional (P.name --| P.$$$ ":") "dom" -- P.term --| P.$$$ ")"))
       >> (fn (name,dom) =>
	      Toplevel.print o Toplevel.theory_to_proof (fundef_setup_termination_proof name dom)));

val _ = OuterSyntax.add_parsers [functionP];
val _ = OuterSyntax.add_parsers [terminationP];


end;


end