Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+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.
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
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip