haftmann [Thu, 26 Apr 2007 13:33:04 +0200] rev 22800
added lemmatas
haftmann [Thu, 26 Apr 2007 13:32:59 +0200] rev 22799
moved code generation pretty integers and characters to separate theories
haftmann [Thu, 26 Apr 2007 13:32:55 +0200] rev 22798
updated doc
wenzelm [Thu, 26 Apr 2007 12:00:12 +0200] rev 22797
mk_const_def: Sign.intern_term (legacy);
wenzelm [Thu, 26 Apr 2007 12:00:05 +0200] rev 22796
renamed some old names Theory.xxx to Sign.xxx;
wenzelm [Thu, 26 Apr 2007 12:00:01 +0200] rev 22795
updated;
narboux [Wed, 25 Apr 2007 21:29:14 +0200] rev 22794
add the lemma supp_eqvt and put the right attribute
nipkow [Wed, 25 Apr 2007 17:50:48 +0200] rev 22793
new lemma splice_length
narboux [Wed, 25 Apr 2007 15:38:56 +0200] rev 22792
fix sml compilation
berghofe [Wed, 25 Apr 2007 15:26:01 +0200] rev 22791
Moved function params_of to inductive_package.ML.
berghofe [Wed, 25 Apr 2007 15:25:22 +0200] rev 22790
Moved functions infer_intro_vars, arities_of, params_of, and
partition_rules to inductive_package.ML.
berghofe [Wed, 25 Apr 2007 15:24:15 +0200] rev 22789
Added functions arities_of, params_of, partition_rules, and
infer_intro_vars (from inductive_realizer.ML).
berghofe [Wed, 25 Apr 2007 15:22:57 +0200] rev 22788
eqvt_tac now instantiates introduction rules before applying them.
narboux [Tue, 24 Apr 2007 18:06:04 +0200] rev 22787
update fresh_fun_simp for debugging purposes
narboux [Tue, 24 Apr 2007 17:16:55 +0200] rev 22786
fixes last commit
narboux [Tue, 24 Apr 2007 16:44:11 +0200] rev 22785
add two lemmas dealing with freshness on permutations.
berghofe [Tue, 24 Apr 2007 15:19:33 +0200] rev 22784
Added datatype_case.ML and nominal_fresh_fun.ML.
berghofe [Tue, 24 Apr 2007 15:18:42 +0200] rev 22783
Added datatype_case.
berghofe [Tue, 24 Apr 2007 15:18:09 +0200] rev 22782
Added intro / elim rules for prod_case.
berghofe [Tue, 24 Apr 2007 15:17:22 +0200] rev 22781
sum_case is now authentic.
berghofe [Tue, 24 Apr 2007 15:15:52 +0200] rev 22780
Adapted to new parse translation for case expressions.
berghofe [Tue, 24 Apr 2007 15:14:31 +0200] rev 22779
Parse / print translations for nested case expressions, taken
from Konrad Slind's TFL package.
berghofe [Tue, 24 Apr 2007 15:13:19 +0200] rev 22778
Streamlined datatype_codegen function using new datatype_of_case
and datatype_of_constr functions.
berghofe [Tue, 24 Apr 2007 15:11:07 +0200] rev 22777
- Moved parse / print translations for case to datatype_case.ML
- Added new functions datatype_of_constr and datatype_of_case
to retrieve datatype corresponding to name of constructor
or case combinator.
berghofe [Tue, 24 Apr 2007 15:07:27 +0200] rev 22776
case constants are now authentic.
narboux [Tue, 24 Apr 2007 14:02:16 +0200] rev 22775
oups : wrong commit
narboux [Tue, 24 Apr 2007 14:01:23 +0200] rev 22774
adds op in front of an infix to fix SML compilation
wenzelm [Mon, 23 Apr 2007 20:44:12 +0200] rev 22773
sane version of read_termTs (proper freeze);
added read_terms, cert_terms;
wenzelm [Mon, 23 Apr 2007 20:44:11 +0200] rev 22772
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
gen_prep_registration: removed unused read_terms (dead code!);
tuned;
wenzelm [Mon, 23 Apr 2007 20:44:10 +0200] rev 22771
added paramify_vars;
infer: replace params uniformly (notably freeze);
wenzelm [Mon, 23 Apr 2007 20:44:09 +0200] rev 22770
def_simproc(_i): proper ProofContext.read/cert_terms;
wenzelm [Mon, 23 Apr 2007 20:44:08 +0200] rev 22769
simplified ProofContext.read_termTs;
urbanc [Mon, 23 Apr 2007 18:38:42 +0200] rev 22768
simplified the proof of pt_set_eqvt (as suggested by Randy Pollack)
haftmann [Mon, 23 Apr 2007 16:38:40 +0200] rev 22767
initial commit
huffman [Sat, 21 Apr 2007 19:32:32 +0200] rev 22766
faster proof of wf_eq_minimal
wenzelm [Sat, 21 Apr 2007 11:07:45 +0200] rev 22765
export get_sort (belongs to Syntax module);
wenzelm [Sat, 21 Apr 2007 11:07:44 +0200] rev 22764
TypeExt.decode_term;
wenzelm [Sat, 21 Apr 2007 11:07:42 +0200] rev 22763
added decode_term (belongs to Syntax module);
urbanc [Sat, 21 Apr 2007 01:34:15 +0200] rev 22762
tuned the setup of fresh_fun
haftmann [Fri, 20 Apr 2007 17:58:27 +0200] rev 22761
defs are added to code data
haftmann [Fri, 20 Apr 2007 17:58:26 +0200] rev 22760
repaired value restriction problem
haftmann [Fri, 20 Apr 2007 17:58:25 +0200] rev 22759
reverted to classical syntax for K_record
haftmann [Fri, 20 Apr 2007 17:58:24 +0200] rev 22758
tuned
ballarin [Fri, 20 Apr 2007 16:55:38 +0200] rev 22757
Interpretation equations applied to attributes
ballarin [Fri, 20 Apr 2007 16:54:57 +0200] rev 22756
Interpretation equations applied to attributes;
code cleanup in read_instantiations
berghofe [Fri, 20 Apr 2007 16:11:17 +0200] rev 22755
Modified eqvt_tac to avoid failure due to introduction rules
whose premises contain variables that do not occur in the
conclusion.
haftmann [Fri, 20 Apr 2007 15:13:06 +0200] rev 22754
clarifed
narboux [Fri, 20 Apr 2007 14:30:35 +0200] rev 22753
modify fresh_fun_simp to ease debugging
haftmann [Fri, 20 Apr 2007 13:30:51 +0200] rev 22752
updated code generator
haftmann [Fri, 20 Apr 2007 13:11:47 +0200] rev 22751
updated
haftmann [Fri, 20 Apr 2007 11:21:53 +0200] rev 22750
adds extracted program to code theorem table
haftmann [Fri, 20 Apr 2007 11:21:52 +0200] rev 22749
unfold attribute now also accepts HOL equations
haftmann [Fri, 20 Apr 2007 11:21:50 +0200] rev 22748
added more stuff
haftmann [Fri, 20 Apr 2007 11:21:49 +0200] rev 22747
add definitions explicitly to code generator table
haftmann [Fri, 20 Apr 2007 11:21:48 +0200] rev 22746
cleared dead code
haftmann [Fri, 20 Apr 2007 11:21:47 +0200] rev 22745
moved axclass module closer to core system
haftmann [Fri, 20 Apr 2007 11:21:42 +0200] rev 22744
Isar definitions are now added explicitly to code theorem table
haftmann [Fri, 20 Apr 2007 11:21:41 +0200] rev 22743
improved case unfolding
haftmann [Fri, 20 Apr 2007 11:21:40 +0200] rev 22742
switched from recdef to function package; constants add, mul, pow now curried; infix syntax for algebraic operations.
haftmann [Fri, 20 Apr 2007 11:21:39 +0200] rev 22741
tuned syntax: K_record is now an authentic constant
haftmann [Fri, 20 Apr 2007 11:21:38 +0200] rev 22740
tuned: now using function package
haftmann [Fri, 20 Apr 2007 11:21:37 +0200] rev 22739
transfer_tac accepts also HOL equations as theorems
haftmann [Fri, 20 Apr 2007 11:21:36 +0200] rev 22738
shifted min/max to class order
haftmann [Fri, 20 Apr 2007 11:21:35 +0200] rev 22737
tuned
haftmann [Fri, 20 Apr 2007 11:21:34 +0200] rev 22736
added class tutorial
haftmann [Fri, 20 Apr 2007 11:21:33 +0200] rev 22735
code generator changes
krauss [Fri, 20 Apr 2007 10:09:32 +0200] rev 22734
generate page labels
krauss [Fri, 20 Apr 2007 10:06:11 +0200] rev 22733
definition lookup via terms, not names. Methods "relation" and "lexicographic_order"
do not depend on "termination" setup.
urbanc [Fri, 20 Apr 2007 00:28:07 +0200] rev 22732
declared lemmas true_eqvt and false_eqvt to be equivariant (suggested by samth at ccs.neu.edu)
paulson [Thu, 19 Apr 2007 18:23:11 +0200] rev 22731
trying to make single-step proofs work better, especially if they contain
abstraction functions. Uniform names for Skolem and Abstraction functions
berghofe [Thu, 19 Apr 2007 16:38:59 +0200] rev 22730
nominal_inductive no longer proves equivariance.
narboux [Thu, 19 Apr 2007 16:27:53 +0200] rev 22729
add a tactic to generate fresh names
wenzelm [Wed, 18 Apr 2007 21:30:14 +0200] rev 22728
simplified ProofContext.infer_types(_pats);
dixon [Wed, 18 Apr 2007 16:23:31 +0200] rev 22727
Improved comments.
krauss [Wed, 18 Apr 2007 11:47:08 +0200] rev 22726
proper header, added regression tests
krauss [Wed, 18 Apr 2007 11:37:43 +0200] rev 22725
added temporary hack to avoid schematic goals in "termination".
paulson [Wed, 18 Apr 2007 11:14:09 +0200] rev 22724
Fixes for proof reconstruction, especially involving abstractions and definitions
wenzelm [Tue, 17 Apr 2007 21:06:59 +0200] rev 22723
export is_dummy_pattern;
huffman [Tue, 17 Apr 2007 03:13:38 +0200] rev 22722
lemma isCont_inv_fun is same as isCont_inverse_function
huffman [Tue, 17 Apr 2007 00:55:00 +0200] rev 22721
moved root and sqrt lemmas from Transcendental.thy to NthRoot.thy
huffman [Tue, 17 Apr 2007 00:37:14 +0200] rev 22720
remove use of pos_boundedE
huffman [Tue, 17 Apr 2007 00:33:49 +0200] rev 22719
lemma geometric_sum no longer needs class division_by_zero
wenzelm [Tue, 17 Apr 2007 00:30:44 +0200] rev 22718
tuned proofs;
haftmann [Mon, 16 Apr 2007 16:11:03 +0200] rev 22717
canonical merge operations
wenzelm [Mon, 16 Apr 2007 12:16:11 +0200] rev 22716
added print_indexname;
tuned;
urbanc [Mon, 16 Apr 2007 07:32:23 +0200] rev 22715
improved the equivariance lemmas for the quantifiers; had to export the lemma eqvt_force_add and eqvt_force_del in the thmdecls
urbanc [Mon, 16 Apr 2007 06:45:22 +0200] rev 22714
added a more usuable lemma for dealing with fresh_fun
huffman [Mon, 16 Apr 2007 04:02:15 +0200] rev 22713
generalized type of lemma geometric_sum
wenzelm [Sun, 15 Apr 2007 23:25:55 +0200] rev 22712
replaced read_term_legacy by read_prop_legacy;
read: intern_skolem before type-inference (many workarounds!);
read: reject_tvars;
removed obsolete TypeInfer.logicT -- use dummyT;
add_fixes: not constraints for external names;
wenzelm [Sun, 15 Apr 2007 23:25:54 +0200] rev 22711
removed obsolete redeclare_skolems;
wenzelm [Sun, 15 Apr 2007 23:25:52 +0200] rev 22710
read prop as prop, not term;
wenzelm [Sun, 15 Apr 2007 23:25:50 +0200] rev 22709
removed obsolete TypeInfer.logicT -- use dummyT;
wenzelm [Sun, 15 Apr 2007 23:25:49 +0200] rev 22708
avoid internal names;
wenzelm [Sun, 15 Apr 2007 14:32:55 +0200] rev 22707
tuned;
wenzelm [Sun, 15 Apr 2007 14:32:07 +0200] rev 22706
legacy_infer_term/prop -- including intern_term;
wenzelm [Sun, 15 Apr 2007 14:32:05 +0200] rev 22705
Thm.plain_prop_of;