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.
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
signature: eqtype to accomodate Alice;
2007-04-03, by wenzelm
renamed comp to compose (avoid clash with Alice keywords);
2007-04-03, by wenzelm
renamed of_sort_derivation record fields (avoid clash with Alice keywords);
2007-04-03, by wenzelm
added ML-Systems/alice.ML;
2007-04-03, by wenzelm
renamed Variable.import to import_thms (avoid clash with Alice keywords);
2007-04-03, by wenzelm
removed assert/deny (avoid clash with Alice keywords and confusion due to strict evaluation);
2007-04-03, by wenzelm
ranamed CodegenData.lazy to lazy_thms (avoid clash with Alice keywords);
2007-04-03, by wenzelm
remove the lemma swap_fun which was not needed
2007-04-03, by narboux
slighltly improved the proof of unicity
2007-04-03, by narboux
Compatibility file for Alice 1.3 -- experimental!
2007-04-03, by wenzelm
rename bij and fresh into bijs and freshs and lookup for eqvts lemma using the ml value instead of the name
2007-04-02, by narboux
optimizing the null instantiation case
2007-04-02, by paulson
now exports distinct_subgoal_tac (needed by MetisAPI)
2007-04-02, by paulson
exception handling
2007-04-02, by paulson
added reserved words mod, div for SML
2007-04-01, by haftmann
added pt_bij' to the collection perm_swap and also added abs_perm to the collection of equivariance lemmas
2007-03-31, by urbanc
Fixed bug in dest_prem: premises of the form "p x_1 ... x_n"
2007-03-31, by berghofe
fixed typo
2007-03-31, by haftmann
simplified constant representation in code generator
2007-03-30, by haftmann
tuned
2007-03-30, by haftmann
equality on strings
2007-03-30, by haftmann
paraphrasing equality
2007-03-30, by haftmann
updated
2007-03-30, by haftmann
improved character output for SML
2007-03-29, by haftmann
dropped legacy ML bindings
2007-03-29, by haftmann
simplified some steps
2007-03-29, by paulson
MESON tactical takes an additional argument: the clausification function.
2007-03-29, by paulson
Now checks for types-only clause before outputting.
2007-03-29, by paulson
- Improved error messages in equivariance proof
2007-03-28, by berghofe
Renamed induct(s)_weak to weak_induct(s) in order to unify
2007-03-28, by berghofe
- Renamed <predicate>_eqvt to <predicate>.eqvt
2007-03-28, by berghofe
the name for the collection of equivariance lemmas is now eqvts (changed from eqvt) in order to avoid clashes with eqvt-lemmas generated in nominal_inductive
2007-03-28, by urbanc
adapted to new nominal_inductive
2007-03-28, by urbanc
Improved code generator for characters: now handles
2007-03-28, by berghofe
tuned proofs (taking full advantage of nominal_inductive)
2007-03-28, by urbanc
adapted to nominal_inductive infrastructure
2007-03-28, by urbanc
made the type sets instance of the "cp" type-class
2007-03-28, by urbanc
added extended the lemma for equivariance of freshness
2007-03-27, by urbanc
adapted to nominal_inductive
2007-03-27, by urbanc
adapted to new nominal_inductive infrastructure
2007-03-27, by urbanc
Adapted to new syntax of nominal_inductive.
2007-03-27, by berghofe
Adapted to changes in nominal_inductive.
2007-03-27, by berghofe
Implemented proof of strong induction rule.
2007-03-27, by berghofe
Exported perm_of_pair, mk_not_sym, and perm_simproc.
2007-03-27, by berghofe
cleaned up HOL/ex/Code*.thy
2007-03-27, by haftmann
fixed document preparation
2007-03-27, by haftmann
fixed problem with mutual recursion
2007-03-26, by krauss
cleaned up Library/ and ex/
2007-03-26, by haftmann
minimal intro rules
2007-03-26, by haftmann
exported interface for intro rules
2007-03-26, by haftmann
moved Eval theory to library
2007-03-26, by haftmann
Eval theory
2007-03-26, by haftmann
tuned
2007-03-26, by haftmann
importing Eval theory
2007-03-26, by haftmann
naming tuned
2007-03-26, by haftmann
cleaned up Library( and ex/
2007-03-26, by haftmann
Clause cache is now in theory data.
2007-03-26, by paulson
"generalize" now replaces ugly mes_XXX generated symbols by 1-letter identifiers.
2007-03-26, by paulson
moving lemmas into appropriate sections
2007-03-25, by urbanc
fixed typing bug in generated code
2007-03-23, by haftmann
fixed typing bug in generated code
2007-03-23, by haftmann
added the permutation operation on options to the list of equivariance lemmas
2007-03-23, by urbanc
dropped
2007-03-23, by haftmann
added empty cases
2007-03-23, by haftmann
added concept for term constructors
2007-03-23, by haftmann
tuned
2007-03-23, by haftmann
two further properties about lists
2007-03-23, by haftmann
removed outdated example
2007-03-23, by haftmann
fixed typo
2007-03-23, by haftmann
added some sketches about library functions
2007-03-23, by haftmann
fixed function syntax
2007-03-22, by krauss
fixed function syntax
2007-03-22, by krauss
corrected the lemmas min_nat_eqvt and min_int_eqvt
2007-03-22, by urbanc
fixed code generator setup
2007-03-22, by haftmann
made function syntax strict, requiring | to separate equations; cleanup
2007-03-22, by krauss
fixed problem with the construction of mutual simp rules
2007-03-22, by krauss
cleanup
2007-03-22, by krauss
clarified an error-message
2007-03-22, by urbanc
tuned some proofs
2007-03-22, by urbanc
added another rule for simultaneous induction, and lemmas for zip
2007-03-21, by krauss
Unified function syntax
2007-03-21, by krauss
Numerous bug fixes. Type clauses distinguished from empty clauses. Working proof reduction.
2007-03-21, by paulson
added example file
2007-03-21, by haftmann
Better documentation path rewriting for src dir, used in tarball build.
2007-03-20, by gagern
Changed AnnoMaLy build process from CVS to tarball sources.
2007-03-20, by gagern
simplified "eval" oracle method
2007-03-20, by krauss
updated keywords
2007-03-20, by haftmann
added theory dependency graph
2007-03-20, by haftmann
improved treatment of defining equations stemming from specification tools
2007-03-20, by haftmann
added instance for lattice
2007-03-20, by haftmann
dropped OrderedGroup.ML
2007-03-20, by haftmann
added class "default" and expansion axioms for undefined
2007-03-20, by haftmann
switched exception from arbitrary to undefined
2007-03-20, by haftmann
updated code generation sections
2007-03-20, by haftmann
fixed typo
2007-03-20, by haftmann
new lemmas
2007-03-20, by haftmann
pretty function arrow for diag serializer
2007-03-20, by haftmann
adjusted definition of defining equation
2007-03-20, by haftmann
fixed slip
2007-03-20, by haftmann
explizit "type" superclass
2007-03-20, by haftmann
tuned the proof
2007-03-19, by urbanc
Removal of axiom names from the theorem cache
2007-03-19, by paulson
No label on "show"; tries to remove dependencies more cleanly
2007-03-19, by paulson
dropped overwrite_warn
2007-03-19, by haftmann
moved Output.overwrite_warn here
2007-03-19, by haftmann
TrueElim and notTrueElim tested and added as safe elim rules.
2007-03-18, by dixon
dropped LOrder.thy in favor of Lattices.thy
2007-03-16, by haftmann
dropped LOrder.thy
2007-03-16, by haftmann
added "satisfies" interface
2007-03-16, by haftmann
dropping dead code
2007-03-16, by haftmann
clarified check of defining equations
2007-03-16, by haftmann
adjusted qualified thm reference
2007-03-16, by haftmann
inf_fun_eq and inf_bool_eq now with meta equality
2007-03-16, by haftmann
added "class"es
2007-03-16, by haftmann
tuned
2007-03-16, by haftmann
dropped superfluous hide
2007-03-16, by haftmann
added lattice definitions
2007-03-16, by haftmann
added instance of sets as distributive lattices
2007-03-16, by haftmann
integrated with LOrder.thy
2007-03-16, by haftmann
moved lattice instance here
2007-03-16, by haftmann
adjusted to new lattice theory developement in Lattices.thy / FixedPoint.thy
2007-03-16, by haftmann
added FIXME hints
2007-03-16, by haftmann
lattice cleanup
2007-03-16, by haftmann
updated
2007-03-16, by haftmann
adjusted for the example file SOS.thy
2007-03-16, by urbanc
added formalisations of typical SOS-proofs
2007-03-16, by urbanc
added eqvt-lemmas for integers and eqvt-tagged the lemma append_eqvt
2007-03-16, by urbanc
removed safe elim flag of trueElim and notFalseElim for testing.
2007-03-16, by dixon
added safe intro rules for removing "True" subgoals as well as "~ False" ones.
2007-03-16, by dixon
move sqrt_divide_self_eq to NthRoot.thy
2007-03-14, by huffman
move bounded (bi)linear operator locales from Lim.thy to RealVector.thy
2007-03-14, by huffman
is_nnf/is_cnf added, defcnf does nothing now if the formula already is in CNF
2007-03-14, by webertj
deleted function for defining candidates and used nominal_primrec instead
2007-03-13, by urbanc
syntax: proper body priorty for derived binders;
2007-03-12, by wenzelm
tuned;
2007-03-12, by wenzelm
removes some unused code that used to try to derive a simpler version of the eqvt lemmas
2007-03-12, by narboux
Adapted to new inductive definition package.
2007-03-12, by berghofe
clarified code
2007-03-11, by haftmann
- Replaced fold by fold_rev to make sure that list of predicate
2007-03-10, by berghofe
- Changed format of descriptor contained in nominal_datatype_info
2007-03-10, by berghofe
Renamed INF to INFM to avoid clash with INF operator defined in FixedPoint theory.
2007-03-10, by berghofe
Adapted to changes in definition of SUP.
2007-03-10, by berghofe
Generalized version of SUP and INF (with index set).
2007-03-10, by berghofe
Eta-expanded codetype_hook to make SML/NJ happy.
2007-03-10, by berghofe
First stab at reconstructing HO problems
2007-03-09, by paulson
constant names now dependent on executable content
2007-03-09, by haftmann
resolved name clashes
2007-03-09, by haftmann
moved order on functions here
2007-03-09, by haftmann
*** empty log message ***
2007-03-09, by haftmann
dropped code datatype certificates
2007-03-09, by haftmann
stepping towards uniform lattice theory development in HOL
2007-03-09, by haftmann
correct typo in latex output
2007-03-06, by narboux
updated this file to the new infrastructure
2007-03-06, by urbanc
fixed function package bug in the handling of multiple guards
2007-03-06, by krauss
major update of the nominal package; there is now an infrastructure
2007-03-06, by urbanc
fix wrong default for find_theorems
2007-03-06, by kleing
document find_theorems syntax change
2007-03-06, by kleing
find_theorems: moved with_dup into the brackets, i.e.
2007-03-06, by kleing
an O(n log n) version of removing duplicates
2007-03-06, by kleing
clean up var/running dir before spawning new tests
2007-03-05, by kleing
additional settings for isatest runs on various platforms
2007-03-05, by kleing
adjust paths
2007-03-05, by kleing
moved all isatest/cron job related files to own directory
2007-03-05, by kleing
AnnoMaLy related files, as discussed in mails with Gerwin Klein
2007-03-05, by gagern
Simplify print mode. Support setproverflag.
2007-03-03, by aspinall
Update test for new parse result
2007-03-03, by aspinall
Add setproverflag, to replace other flag controls
2007-03-03, by aspinall
Add objtypes to openblock/closeblock and theory items (can be used to control folding).
2007-03-03, by aspinall
Add more attributes to openblock. Change theory item objtype field to proper objtype.
2007-03-03, by aspinall
Add Isabelle-specific objtypes
2007-03-03, by aspinall
Comment
2007-03-03, by aspinall
clarified code
2007-03-03, by haftmann
clarified error message
2007-03-03, by haftmann
moved instance option :: finite to Finite_Set.thy
2007-03-03, by haftmann
moved instance option :: finite here
2007-03-03, by haftmann
Fix idvalue output and PGML print mode raw encode/decode.
2007-03-03, by aspinall
permitting empty datatypes
2007-03-02, by haftmann
improved handling of nat numerals
2007-03-02, by haftmann
tuned code theorems for ord on integers
2007-03-02, by haftmann
simplified code generator setup
2007-03-02, by haftmann
tuned code theorems
2007-03-02, by haftmann
added add_numerals_of
2007-03-02, by haftmann
now using "class"
2007-03-02, by haftmann
using "fst" "snd" for Haskell code
2007-03-02, by haftmann
added code theorems for UNIV
2007-03-02, by haftmann
adjusted to latest changes
2007-03-02, by haftmann
new code theorems
2007-03-02, by haftmann
syntax for "class attach const"
2007-03-02, by haftmann
prefix of class interpretation not mandatory any longer
2007-03-02, by haftmann
Meson.is_fol_term now takes a theory as argument. Minor tidying.
2007-03-02, by paulson
New code to store theorem names in a concise form rather than as fully-qualified.
2007-03-02, by paulson
The first-order test now tests for the obscure case of a polymorphic constant like 1 being
2007-03-02, by paulson
abbrev: be permissive after transformation;
2007-02-28, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip