doc/Contents
author Timothy Bourke
Mon, 09 Feb 2009 17:25:07 +1100
changeset 29848 a7c164e228e1
parent 25248 cc5cf5f1178b
child 29747 bab2371e0348
child 30240 5b25fee0362c
permissions -rw-r--r--
Nicer names in FindTheorems. * Patch NameSpace.get_accesses, contributed by Timothy Bourke: NameSpace.get_accesses has been patched to fix the following bug: theory OverHOL imports Main begin lemma conjI: "a & b --> b" by blast ML {* val ns = PureThy.facts_of @{theory} |> Facts.space_of; val x1 = NameSpace.get_accesses ns "HOL.conjI"; val x2 = NameSpace.get_accesses ns "OverHOL.conjI"; *} end where x1 = ["conjI", "HOL.conjI"] and x2 = ["conjI", "OverHOL.conjI"], but x1 should be just ["HOL.conjI"]. NameSpace.get_accesses is only used within the NameSpace structure itself. The two uses have been modified to retain their original behaviour. Note that NameSpace.valid_accesses gives different results: get_accesses ns "HOL.eq_class.eq" gives ["eq", "eq_class.eq", "HOL.eq_class.eq"] but, valid_accesses ns "HOL.eq_class.eq" gives ["HOL.eq_class.eq", "eq_class.eq", "HOL.eq", "eq"] * Patch FindTheorems: Prefer names that are shorter to type in the current context. * Re-export space_of.

Learning and using Isabelle
  tutorial        Tutorial on Isabelle/HOL
  isar-overview   Tutorial on Isar
  locales         Tutorial on Locales
  classes         Tutorial on Type Classes
  functions       Tutorial on Function Definitions
  codegen         Tutorial on Code Generation
  sugar           LaTeX sugar for proof documents
  ind-defs        (Co)Inductive Definitions in ZF

Reference Manuals
  isar-ref        The Isabelle/Isar Reference Manual
  implementation  The Isabelle/Isar Implementation Manual
  system          The Isabelle System Manual
  ref             The Isabelle Reference Manual
  logics          Isabelle's Logics: overview and misc logics
  logics-HOL      Isabelle's Logics: HOL
  logics-ZF       Isabelle's Logics: FOL and ZF