Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
renamed some old names Theory.xxx to Sign.xxx;
2007-04-26, by wenzelm
updated;
2007-04-26, by wenzelm
add the lemma supp_eqvt and put the right attribute
2007-04-25, by narboux
new lemma splice_length
2007-04-25, by nipkow
fix sml compilation
2007-04-25, by narboux
Moved function params_of to inductive_package.ML.
2007-04-25, by berghofe
Moved functions infer_intro_vars, arities_of, params_of, and
2007-04-25, by berghofe
Added functions arities_of, params_of, partition_rules, and
2007-04-25, by berghofe
eqvt_tac now instantiates introduction rules before applying them.
2007-04-25, by berghofe
update fresh_fun_simp for debugging purposes
2007-04-24, by narboux
fixes last commit
2007-04-24, by narboux
add two lemmas dealing with freshness on permutations.
2007-04-24, by narboux
Added datatype_case.ML and nominal_fresh_fun.ML.
2007-04-24, by berghofe
Added datatype_case.
2007-04-24, by berghofe
Added intro / elim rules for prod_case.
2007-04-24, by berghofe
sum_case is now authentic.
2007-04-24, by berghofe
Adapted to new parse translation for case expressions.
2007-04-24, by berghofe
Parse / print translations for nested case expressions, taken
2007-04-24, by berghofe
Streamlined datatype_codegen function using new datatype_of_case
2007-04-24, by berghofe
- Moved parse / print translations for case to datatype_case.ML
2007-04-24, by berghofe
case constants are now authentic.
2007-04-24, by berghofe
oups : wrong commit
2007-04-24, by narboux
adds op in front of an infix to fix SML compilation
2007-04-24, by narboux
sane version of read_termTs (proper freeze);
2007-04-23, by wenzelm
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
2007-04-23, by wenzelm
added paramify_vars;
2007-04-23, by wenzelm
def_simproc(_i): proper ProofContext.read/cert_terms;
2007-04-23, by wenzelm
simplified ProofContext.read_termTs;
2007-04-23, by wenzelm
simplified the proof of pt_set_eqvt (as suggested by Randy Pollack)
2007-04-23, by urbanc
initial commit
2007-04-23, by haftmann
faster proof of wf_eq_minimal
2007-04-21, by huffman
export get_sort (belongs to Syntax module);
2007-04-21, by wenzelm
TypeExt.decode_term;
2007-04-21, by wenzelm
added decode_term (belongs to Syntax module);
2007-04-21, by wenzelm
tuned the setup of fresh_fun
2007-04-21, by urbanc
defs are added to code data
2007-04-20, by haftmann
repaired value restriction problem
2007-04-20, by haftmann
reverted to classical syntax for K_record
2007-04-20, by haftmann
tuned
2007-04-20, by haftmann
Interpretation equations applied to attributes
2007-04-20, by ballarin
Interpretation equations applied to attributes;
2007-04-20, by ballarin
Modified eqvt_tac to avoid failure due to introduction rules
2007-04-20, by berghofe
clarifed
2007-04-20, by haftmann
modify fresh_fun_simp to ease debugging
2007-04-20, by narboux
updated code generator
2007-04-20, by haftmann
updated
2007-04-20, by haftmann
adds extracted program to code theorem table
2007-04-20, by haftmann
unfold attribute now also accepts HOL equations
2007-04-20, by haftmann
added more stuff
2007-04-20, by haftmann
add definitions explicitly to code generator table
2007-04-20, by haftmann
cleared dead code
2007-04-20, by haftmann
moved axclass module closer to core system
2007-04-20, by haftmann
Isar definitions are now added explicitly to code theorem table
2007-04-20, by haftmann
improved case unfolding
2007-04-20, by haftmann
switched from recdef to function package; constants add, mul, pow now curried; infix syntax for algebraic operations.
2007-04-20, by haftmann
tuned syntax: K_record is now an authentic constant
2007-04-20, by haftmann
tuned: now using function package
2007-04-20, by haftmann
transfer_tac accepts also HOL equations as theorems
2007-04-20, by haftmann
shifted min/max to class order
2007-04-20, by haftmann
tuned
2007-04-20, by haftmann
added class tutorial
2007-04-20, by haftmann
code generator changes
2007-04-20, by haftmann
generate page labels
2007-04-20, by krauss
definition lookup via terms, not names. Methods "relation" and "lexicographic_order"
2007-04-20, by krauss
declared lemmas true_eqvt and false_eqvt to be equivariant (suggested by samth at ccs.neu.edu)
2007-04-20, by urbanc
trying to make single-step proofs work better, especially if they contain
2007-04-19, by paulson
nominal_inductive no longer proves equivariance.
2007-04-19, by berghofe
add a tactic to generate fresh names
2007-04-19, by narboux
simplified ProofContext.infer_types(_pats);
2007-04-18, by wenzelm
Improved comments.
2007-04-18, by dixon
proper header, added regression tests
2007-04-18, by krauss
added temporary hack to avoid schematic goals in "termination".
2007-04-18, by krauss
Fixes for proof reconstruction, especially involving abstractions and definitions
2007-04-18, by paulson
export is_dummy_pattern;
2007-04-17, by wenzelm
lemma isCont_inv_fun is same as isCont_inverse_function
2007-04-17, by huffman
moved root and sqrt lemmas from Transcendental.thy to NthRoot.thy
2007-04-17, by huffman
remove use of pos_boundedE
2007-04-17, by huffman
lemma geometric_sum no longer needs class division_by_zero
2007-04-17, by huffman
tuned proofs;
2007-04-17, by wenzelm
canonical merge operations
2007-04-16, by haftmann
added print_indexname;
2007-04-16, by wenzelm
improved the equivariance lemmas for the quantifiers; had to export the lemma eqvt_force_add and eqvt_force_del in the thmdecls
2007-04-16, by urbanc
added a more usuable lemma for dealing with fresh_fun
2007-04-16, by urbanc
generalized type of lemma geometric_sum
2007-04-16, by huffman
replaced read_term_legacy by read_prop_legacy;
2007-04-15, by wenzelm
removed obsolete redeclare_skolems;
2007-04-15, by wenzelm
read prop as prop, not term;
2007-04-15, by wenzelm
removed obsolete TypeInfer.logicT -- use dummyT;
2007-04-15, by wenzelm
avoid internal names;
2007-04-15, by wenzelm
tuned;
2007-04-15, by wenzelm
legacy_infer_term/prop -- including intern_term;
2007-04-15, by wenzelm
Thm.plain_prop_of;
2007-04-15, by wenzelm
added decode_types (from type_infer.ML);
2007-04-15, by wenzelm
added read_term;
2007-04-15, by wenzelm
added mixfixT (from type_infer.ML);
2007-04-15, by wenzelm
proper interface infer_types(_pat);
2007-04-15, by wenzelm
Thm.fold_terms;
2007-04-15, by wenzelm
removed unused Output.panic hook -- internal to PG wrapper;
2007-04-15, by wenzelm
moved get_sort to sign.ML;
2007-04-15, by wenzelm
removed obsolete inferT_axm;
2007-04-15, by wenzelm
removed obsolete infer_types(_simult);
2007-04-15, by wenzelm
moved Drule.plain_prop_of, Drule.fold_terms to more_thm.ML;
2007-04-15, by wenzelm
load type_infer.ML early;
2007-04-15, by wenzelm
adapted decode_type;
2007-04-15, by wenzelm
proper ProofContext.infer_types;
2007-04-15, by wenzelm
Thm.fold_terms;
2007-04-15, by wenzelm
replaced axioms/finalconsts by proper axiomatization;
2007-04-15, by wenzelm
simplified read_axm;
2007-04-14, by wenzelm
tuned comment;
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
removed redundant string_of_vname (see term.ML);
2007-04-14, by wenzelm
removed obsolete read_ctyp, read_def_cterm;
2007-04-14, by wenzelm
tuned signature;
2007-04-14, by wenzelm
read_typ_XXX: no sorts;
2007-04-14, by wenzelm
added read_def_cterms, read_cterm (from thm.ML);
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
removed Pure/Syntax/ROOT.ML;
2007-04-14, by wenzelm
Term.string_of_vname;
2007-04-14, by wenzelm
Theory.inferT_axm;
2007-04-14, by wenzelm
do not enable Toplevel.debug globally;
2007-04-14, by wenzelm
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
2007-04-14, by wenzelm
canonical merge operations
2007-04-14, by haftmann
declarations: apply target_morphism;
2007-04-14, by wenzelm
inst(T)_morphism: avoid reference to static theory value;
2007-04-14, by wenzelm
tuned signature;
2007-04-14, by wenzelm
added Morphism.transform/form (generic non-sense);
2007-04-14, by wenzelm
Morphism.transform/form;
2007-04-14, by wenzelm
data declaration: removed obsolete target_morphism (still required for local data!?);
2007-04-14, by wenzelm
data declaration: removed obsolete target_morphism;
2007-04-14, by wenzelm
added eval_antiquotes_fn (tmp);
2007-04-13, by wenzelm
tuned document (headers, sections, spacing);
2007-04-13, by wenzelm
do translation: CONST;
2007-04-13, by wenzelm
eval_antiquotes: proper parentheses for projection;
2007-04-13, by wenzelm
canonical merge operations
2007-04-13, by haftmann
Removed erroneous application of rev in get_clauses that caused
2007-04-13, by berghofe
more robust proof
2007-04-13, by krauss
Experimental code for the interpretation of definitions.
2007-04-13, by ballarin
Experimental interpretation code for definitions.
2007-04-13, by ballarin
New file for locale regression tests.
2007-04-13, by ballarin
debug versions of finite_guess and fresh_guess do not fail if they can not solve the goal
2007-04-13, by narboux
minimize imports
2007-04-13, by huffman
new simp rule exp_ln; new standard proof of DERIV_exp_ln_one; changed imports
2007-04-13, by huffman
moved nonstandard derivative stuff from Deriv.thy into new file HDeriv.thy
2007-04-13, by huffman
added proj_value_antiq;
2007-04-12, by wenzelm
absdummy: use internal name uu to avoid renaming of popular names;
2007-04-12, by wenzelm
tuned the proof of lemma pt_list_set_fresh (as suggested by Randy Pollack) and tuned the syntax for sub_contexts
2007-04-12, by urbanc
updated;
2007-04-12, by wenzelm
output_basic: added isaantiq markup (only inside verbatim tokens);
2007-04-12, by wenzelm
newenvironment{isaantiq};
2007-04-12, by wenzelm
Zero variable indexes in clauses
2007-04-12, by paulson
Improved treatment of classrel/arity clauses
2007-04-12, by paulson
Fixed the treatment of TVars in conjecture clauses (they are deleted, not frozen)
2007-04-12, by paulson
Improved and simplified the treatment of classrel/arity clauses
2007-04-12, by paulson
canonical merge operations
2007-04-12, by haftmann
moved nonstandard limit stuff from Lim.thy into new theory HLim.thy
2007-04-12, by huffman
run annomaly from makedist
2007-04-12, by kleing
set special ISABELLE_USER_HOME as in other isatest settings
2007-04-12, by isatest
isatest version of annomaly script. to be run from istatest-makedist.
2007-04-12, by kleing
new standard proof of lemma LIM_inverse
2007-04-12, by huffman
new class syntax for scaleR and norm classes
2007-04-11, by huffman
removed debugging code
2007-04-11, by krauss
canonical merge operations
2007-04-11, by haftmann
tuned
2007-04-11, by haftmann
dropped legacy ML bindings
2007-04-11, by haftmann
moved nonstandard stuff from SEQ.thy into new file HSEQ.thy
2007-04-11, by huffman
move lemma real_of_nat_inverse_le_iff from NSA.thy to NthRoot.thy
2007-04-11, by huffman
new standard proof of convergent = Cauchy
2007-04-11, by huffman
new standard proof of LIMSEQ_realpow_zero
2007-04-10, by huffman
new LIM/isCont lemmas for abs, of_real, and power
2007-04-10, by huffman
some restructuring
2007-04-10, by krauss
interpretation bounded_linear_of_real
2007-04-10, by huffman
removed unnecessary premise from power_le_imp_le_base
2007-04-10, by huffman
proper handling of morphisms
2007-04-10, by krauss
Moving "FunDef" up in the HOL development graph, since it is independent from "Recdef" and "Datatype" now.
2007-04-10, by krauss
inline_antiq: no longer forces ML_Syntax.atomic;
2007-04-10, by wenzelm
removed dead code
2007-04-10, by krauss
tuned
2007-04-10, by krauss
added example for definitions in local contexts
2007-04-10, by krauss
removed obsolete workaround
2007-04-10, by krauss
generalized type of lemma setsum_product
2007-04-09, by huffman
new standard proofs of some LIMSEQ lemmas
2007-04-09, by huffman
rearranged sections
2007-04-08, by huffman
remove redundant lemmas
2007-04-08, by huffman
removed obsolete workarounds
2007-04-07, by krauss
deleted remaining instances of swap_simp_a and swap_simp_b (obsolete now)
2007-04-07, by urbanc
tuned slightly the previous commit
2007-04-07, by urbanc
perm_simp can now simplify using the rules (a,b) o a = b and (a,b) o b = a
2007-04-07, by narboux
add new standard proofs for limits of sequences
2007-04-06, by huffman
Replaced add_inductive_i by add_inductive_global.
2007-04-05, by berghofe
- Tried to make name_of_thm more robust against changes of the
2007-04-05, by berghofe
- Removed occurrences of ProofContext.export in add_ind_def that
2007-04-05, by berghofe
thy_deps: sort Context.thy_ord;
2007-04-05, by wenzelm
added thy_ord -- order of creation;
2007-04-05, by wenzelm
simplified thy_deps using Theory.ancestors_of (in order of creation);
2007-04-04, by wenzelm
renamed Variable.importT to importT_thms;
2007-04-04, by wenzelm
removed unused dep_graph;
2007-04-04, by wenzelm
theory: maintain ancestors in order of creation;
2007-04-04, by wenzelm
rep_thm/cterm/ctyp: removed obsolete sign field;
2007-04-04, by wenzelm
rebind HOL.refl as refl (hidden by widen.refl);
2007-04-04, by wenzelm
rep_thm/cterm/ctyp: removed obsolete sign field;
2007-04-04, by wenzelm
make fresh_guess fail if it does not solve the subgoal
2007-04-04, by narboux
add a few details in the Fst and Snd cases of unicity proof
2007-04-04, by narboux
find_first is just an alias
2007-04-04, by paulson
added print_mode (generic non-sense);
2007-04-04, by wenzelm
improved exception CTERM;
2007-04-04, by wenzelm
removed unused info channel;
2007-04-04, by wenzelm
added print_mode;
2007-04-04, by wenzelm
removed unused info channel;
2007-04-04, by wenzelm
renamed Output.has_mode to print_mode_active;
2007-04-04, by wenzelm
tuned comment;
2007-04-04, by wenzelm
cleaned-up Output functions;
2007-04-04, by wenzelm
improved exception CTERM;
2007-04-04, by wenzelm
added scanwords from library.ML (for obsolete rename_tac);
2007-04-04, by wenzelm
removed obsolete scanwords (see obsolete tactic.ML:rename_tac for its only use);
2007-04-04, by wenzelm
removed dead code;
2007-04-04, by wenzelm
cleaned-up Output functions;
2007-04-04, by wenzelm
eliminated obsolete rename_tac;
2007-04-04, by wenzelm
removed obsolete sign_of/sign_of_thm;
2007-04-04, by wenzelm
ML antiquotes;
2007-04-04, by wenzelm
tuned comments;
2007-04-03, by wenzelm
fixed chr/explode;
2007-04-03, by wenzelm
avoid overloaded integer constants (accomodate Alice);
2007-04-03, by wenzelm
avoid clash with Alice keywords;
2007-04-03, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip