# HG changeset patch # User Cezary Kaliszyk # Date 1256800009 -3600 # Node ID fcff14e578d33cbfccd655db57d8d8f20e675407 # Parent 38810e1df801d25e1d3a6eb29b4a934bf146075a Fixed wrong CARD definition and removed the "Does not work anymore" comment. diff -r 38810e1df801 -r fcff14e578d3 FSet.thy --- a/FSet.thy Thu Oct 29 07:29:12 2009 +0100 +++ b/FSet.thy Thu Oct 29 08:06:49 2009 +0100 @@ -177,7 +177,7 @@ term fmap thm fmap_def -ML {* val fset_defs = @{thms EMPTY_def IN_def FUNION_def card_def INSERT_def fmap_def fold_def} *} +ML {* val fset_defs = @{thms EMPTY_def IN_def FUNION_def CARD_def INSERT_def fmap_def fold_def} *} (* ML {* val consts = map (fst o dest_Const o fst o Logic.dest_equals o concl_of) fset_defs *} *) ML {* @@ -187,7 +187,6 @@ @{const_name "map"}]; *} -(* FIXME: does not work anymore :o( *) ML {* val fset_defs_sym = add_lower_defs @{context} fset_defs *} lemma memb_rsp: @@ -315,7 +314,7 @@ @ @{thms ho_all_prs ho_ex_prs} *} ML {* val trans2 = @{thm QUOT_TYPE_I_fset.R_trans2} *} ML {* val reps_same = @{thm QUOT_TYPE_I_fset.REPS_same} *} -ML {* val defs = @{thms EMPTY_def IN_def UNION_def card_def INSERT_def fmap_def fold_def} *} +ML {* val defs = fset_defs *} (* ML {* val consts = map (fst o dest_Const o fst o Logic.dest_equals o concl_of) fset_defs *} *) ML {* val consts = [@{const_name "Nil"}, @{const_name "Cons"}, diff -r 38810e1df801 -r fcff14e578d3 LamEx.thy --- a/LamEx.thy Thu Oct 29 07:29:12 2009 +0100 +++ b/LamEx.thy Thu Oct 29 08:06:49 2009 +0100 @@ -17,7 +17,6 @@ | a3: "\t \ ([(a,b)]\s); a\[b].s\ \ rLam a t \ rLam b s" quotient lam = rlam / alpha -apply - sorry print_quotients diff -r 38810e1df801 -r fcff14e578d3 isar-keywords-prove.el --- a/isar-keywords-prove.el Thu Oct 29 07:29:12 2009 +0100 +++ b/isar-keywords-prove.el Thu Oct 29 08:06:49 2009 +0100 @@ -335,6 +335,7 @@ "header" "help" "kill_thy" + "nitpick" "normal_form" "pr" "pretty_setmargin" @@ -581,7 +582,6 @@ "apply_end" "back" "defer" - "nitpick" "prefer")) (provide 'isar-keywords)